@@ -23,6 +23,7 @@ open import Reflection.Tactic
2323open import Reflection.AST.Term using (_≟-Pattern_)
2424open import Reflection.Utils
2525open import Reflection.Utils.TCI
26+ open import Reflection.QuotedDefinitions
2627
2728open import Class.DecEq.Core
2829open import Class.Functor
@@ -39,10 +40,6 @@ open ClauseExprM
3940private
4041 instance _ = ContextMonad-MonadTC
4142
42- `yes `no : Term → Term
43- `yes x = quote _because_ ◆⟦ quote true ◆ ∣ quote ofʸ ◆⟦ x ⟧ ⟧
44- `no x = quote _because_ ◆⟦ quote false ◆ ∣ quote ofⁿ ◆⟦ x ⟧ ⟧
45-
4643 -- We take the Dec P argument first to improve type checking performance.
4744 -- It's easy to infer the type of P from this argument and we need to know
4845 -- P to be able to check the pattern lambda generated for the P → Q direction
@@ -77,15 +74,15 @@ private
7774
7875 -- c x1 .. xn ≡ c y1 .. yn ⇔ x1 ≡ y1 .. xn ≡ yn
7976 genEquiv : ℕ → Term
80- genEquiv n = quote mk⇔ ∙⟦ `λ⟦ reflPattern n ⇒ quote refl ◆ ⟧ ∣ `λ⟦ quote refl ◇ ⇒ reflTerm n ⟧ ⟧
77+ genEquiv n = quote mk⇔ ∙⟦ `λ⟦ reflPattern n ⇒ ` refl ⟧ ∣ `λ⟦ `` refl ⇒ reflTerm n ⟧ ⟧
8178 where
8279 reflPattern : ℕ → Pattern
8380 reflPattern 0 = quote tt ◇
84- reflPattern (suc n) = quote _,_ ◇⟦ reflPattern n ∣ quote refl ◇ ⟧
81+ reflPattern (suc n) = quote _,_ ◇⟦ reflPattern n ∣ `` refl ⟧
8582
8683 reflTerm : ℕ → Term
8784 reflTerm 0 = quote tt ◆
88- reflTerm (suc n) = quote _,_ ◆⟦ reflTerm n ∣ quote refl ◆ ⟧
85+ reflTerm (suc n) = quote _,_ ◆⟦ reflTerm n ∣ ` refl ⟧
8986
9087 toMapDiag : SinglePattern → SinglePattern → NE.List⁺ SinglePattern × TC (ClauseExpr ⊎ Maybe Term)
9188 toMapDiag p@(_ , arg _ p₁) p'@(_ , arg _ p₂) =
0 commit comments