agda / agda2hs

Compiling Agda code to readable Haskell

Home Page:https://agda.github.io/agda2hs

Geek Repo:Geek Repo

Github PK Tool:Github PK Tool

Provide Sigma compiled to tuples

flupe opened this issue · comments

record Sigma (a : Set) (b : @0 a  Set) : Set where
  constructor Pair
  field
    fst : a
    snd : b fst
{-# COMPILE AGDA2HS Sigma #-}

(The builtin dependent sigma type, properly annotated).

Looks good. Once we have #105 we could make it compile to actual Haskell pairs.