Skip to content

Commit

Permalink
Use different universe levels.
Browse files Browse the repository at this point in the history
Fixes #1.
  • Loading branch information
gebner committed Dec 1, 2021
1 parent cfcabfe commit e46540e
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions Qq/Macro.lean
Original file line number Diff line number Diff line change
Expand Up @@ -71,8 +71,8 @@ def addSyntaxDollar : Syntax → Syntax
Syntax.ident info rawVal (addDollar val) preresolved
| stx => panic! "addSyntaxDollar {stx}"

def mkAbstractedLevelName (e : Expr) : MetaM Name :=
e.getAppFn.constName?.getD `udummy
def mkAbstractedLevelName (e : Expr) : MetaM Name := do
e.getAppFn.constName?.getD `udummy ++ (← mkFreshId)

def isBad (e : Expr) : Bool := do
if let Expr.const (Name.str _ "rec" _) _ _ := e.getAppFn then
Expand Down

0 comments on commit e46540e

Please sign in to comment.