Skip to content

Commit

Permalink
Fix incorrectly quoted sorts (#7203)
Browse files Browse the repository at this point in the history
  • Loading branch information
UlfNorell committed Mar 25, 2024
1 parent 0b2f857 commit 4eb7f95
Show file tree
Hide file tree
Showing 2 changed files with 16 additions and 2 deletions.
4 changes: 2 additions & 2 deletions src/full/Agda/TypeChecking/Quote.hs
Original file line number Diff line number Diff line change
Expand Up @@ -179,8 +179,8 @@ quotingKit = do
quoteSort PiSort{} = pure unsupportedSort
quoteSort FunSort{} = pure unsupportedSort
quoteSort UnivSort{} = pure unsupportedSort
quoteSort (MetaS x es) = quoteTerm $ MetaV x es
quoteSort (DefS d es) = quoteTerm $ Def d es
quoteSort (MetaS x es) = pure unsupportedSort
quoteSort (DefS d es) = pure unsupportedSort
quoteSort (DummyS s) =__IMPOSSIBLE_VERBOSE__ s

quoteType :: Type -> ReduceM Term
Expand Down
14 changes: 14 additions & 0 deletions test/Succeed/Issue7187.agda
Original file line number Diff line number Diff line change
@@ -0,0 +1,14 @@
open import Agda.Builtin.Reflection renaming (bindTC to _>>=_)
open import Agda.Builtin.Unit
open import Agda.Builtin.Nat
open import Agda.Builtin.List

macro
`Nat : Term TC ⊤
`Nat hole = do
ty inferType hole
_ debugPrint "tactic" 10 (termErr ty ∷ [])
unify hole (def (quote Nat) [])

boom : `Nat
boom = 1

0 comments on commit 4eb7f95

Please sign in to comment.