mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-12-01 09:49:24 +03:00
a972778eab
They don't all pass yet, for minor reasons. Coming shortly... Unfortunately the startup overhead for chez is really noticeable here!
9 lines
312 B
Plaintext
9 lines
312 B
Plaintext
data Eq : $a -> $b -> Type where
|
|
Refl : Eq $x $x
|
|
|
|
okay : {p : $a -> Type} -> (1 x : $a) -> (1 y : $a) -> (1 prf : Eq x y) ->
|
|
p x -> p y
|
|
-- Should fail on the LHS, before even getting to the RHS, because
|
|
-- after elaboration 'x' appears twice even though it is linearly bound.
|
|
okay $x $x Refl $q = q
|