Idris2/tests/idris2/total/positivity004/Issue1771-1.idr
2023-09-07 14:57:22 +01:00

17 lines
224 B
Idris

%default total
data Fix : (Type -> Type) -> Type where
MkFix : f (Fix f) -> Fix f
F : Type
F = Fix Not
yesF : Not F -> F
yesF nf = MkFix nf
notF : Not F
notF (MkFix f) = f (yesF f)
argh : Void
argh = notF (yesF notF)