Skip to content

Commit

Permalink
Fix #16
Browse files Browse the repository at this point in the history
  • Loading branch information
eric-wieser committed Aug 18, 2024
1 parent 71f5442 commit 338ce9d
Show file tree
Hide file tree
Showing 2 changed files with 2 additions and 0 deletions.
1 change: 1 addition & 0 deletions Qq/Macro.lean
Original file line number Diff line number Diff line change
Expand Up @@ -588,6 +588,7 @@ partial def floatExprAntiquot' [Monad m] [MonadQuotation m] (depth : Nat) :
| `(q($x)) => do `(q($(← floatExprAntiquot' (depth + 1) x)))
| `(Type $term) => do `(Type $(← floatLevelAntiquot' term))
| `(Sort $term) => do `(Sort $(← floatLevelAntiquot' term))
| `($n:ident.{$us,*}) => do `($n.{$(← us.getElems.mapM floatLevelAntiquot'),*})
| stx => do
if let (some (kind, _pseudo), false) := (stx.antiquotKind?, stx.isEscapedAntiquot) then
let term := stx.getAntiquotTerm
Expand Down
1 change: 1 addition & 0 deletions Qq/Match.lean
Original file line number Diff line number Diff line change
Expand Up @@ -400,6 +400,7 @@ private partial def floatExprAntiquot (depth : Nat) : Term → StateT (Array (TS
| `(q($x)) => do `(q($(← floatExprAntiquot (depth + 1) x)))
| `(Type $term) => do `(Type $(← floatLevelAntiquot term))
| `(Sort $term) => do `(Sort $(← floatLevelAntiquot term))
| `($n:ident.{$us,*}) => do `($n.{$(← us.getElems.mapM floatLevelAntiquot),*})
| stx => do
if stx.1.isAntiquot && !stx.1.isEscapedAntiquot then
let term : Term := ⟨stx.1.getAntiquotTerm⟩
Expand Down

0 comments on commit 338ce9d

Please sign in to comment.