Idris2/tests/idris2/operators/operators002/Errors3.idr

9 lines
142 B
Idris
Raw Normal View History

2023-10-25 14:01:52 +03:00
typebind infixr 0 =@
0 (=@) : (a : Type) -> (a -> Type) -> Type
(=@) a f = (1 x : a) -> f x
wrongId : {0 a : Type} -> a =@ a
wrongId x = x