Idris2/tests/ttimp/eta002/Eta.yaff
Edwin Brady a972778eab Add test script
They don't all pass yet, for minor reasons. Coming shortly...
Unfortunately the startup overhead for chez is really noticeable here!
2020-05-19 18:25:18 +01:00

17 lines
311 B
Plaintext

data Nat : Type where
Z : Nat
S : Nat -> Nat
plus : Nat -> Nat -> Nat
plus Z $y = y
plus (S $k) $y = S (plus k y)
data Eq : $a -> $b -> Type where
Refl : Eq $x $x
data Test : Type where
MkTest : Integer -> Integer -> Test
etaBad : Eq MkTest (\x : Char => \y => MkTest ? ?)
etaBad = Refl