mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-12-19 09:12:34 +03:00
10 lines
158 B
Idris
10 lines
158 B
Idris
data Foo : Nat -> Type where
|
|
|
|
G : (0 yv : Nat) -> Type
|
|
G yv = Foo yv -> Bool
|
|
|
|
partial
|
|
f : (0 x : Nat) -> Nat
|
|
f x = case G x of
|
|
(Foo x' -> _) => x'
|