Idris2/tests/idris2/reflection016/BindElabScBug.idr

11 lines
133 B
Idris
Raw Normal View History

import Language.Reflection
%default total
f : TTImp -> Elab Nat
f _ = pure 5
%language ElabReflection
x = %runElab quote 4 >>= f