Idris2/tests/idris2/interface/interface021/LocalHint.idr
2023-09-07 14:57:22 +01:00

24 lines
380 B
Idris

Gnu : Type
Gnu = Int
Foo : Type
Foo = Bool
A : Foo
A = True
mkFoo : Gnu -> Foo
mkFoo gnu = A
gnat : {auto startHere : (a : Foo ** a = A)} -> Unit
gnat = ()
pathology : (gnu : Gnu) -> Unit
pathology gnu =
let %hint foo : Foo
foo = mkFoo gnu
%hint bar : Foo -> (ford : arg = A)
-> (a : Foo ** a = A)
bar _ Refl = (A ** Refl)
in gnat