Idris2/tests/idris2/reg/reg038/Test2.idr
2023-09-07 14:57:22 +01:00

10 lines
160 B
Idris

data Foo : Nat -> Type where
0 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'