Issue5789.agda 252 B

123456789101112131415161718
  1. open import Agda.Builtin.List
  2. open import Agda.Builtin.Reflection
  3. open import Agda.Builtin.Unit
  4. postulate
  5. A B : Set
  6. @0 a : A
  7. tac : Term → TC ⊤
  8. tac = unify (def (quote a) [])
  9. postulate
  10. f : {@0 @(tactic tac) x : A} → B
  11. test : B
  12. test = f