Idris2/tests/idris2/operators/operators002/Errors.idr
2024-02-24 12:28:10 +00:00

10 lines
168 B
Idris

typebind infixr 0 =@
0 (=@) : (a : Type) -> (a -> Type) -> Type
(=@) a f = (1 x : a) -> f x
data S : {ty : Type} -> (x : ty) -> Type where
MkS : (x := ty) =@ S x