mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-12-15 22:32:19 +03:00
16 lines
252 B
Idris
16 lines
252 B
Idris
%default total
|
|
|
|
data F : Type where
|
|
MkFix : ((0 g : Type -> Type) -> g === Not -> g F) -> F
|
|
|
|
yesF : Not F -> F
|
|
yesF nf = MkFix (\ g, Refl => nf)
|
|
|
|
notF : Not F
|
|
notF (MkFix f) =
|
|
let g = f Not Refl in
|
|
g (yesF g)
|
|
|
|
argh : Void
|
|
argh = notF (yesF notF)
|