File tree Expand file tree Collapse file tree 3 files changed +3
-3
lines changed
Expand file tree Collapse file tree 3 files changed +3
-3
lines changed Original file line number Diff line number Diff line change @@ -92,7 +92,7 @@ Returns the declaration name.
9292-/
9393def declareTacticSyntax (tactic : Syntax) (name? : Option Name := none) : TermElabM Name :=
9494 withFreshMacroScope do
95- let name ← name?.getDM do MonadQuotation.addMacroScope ((← getEnv).asyncPrefix?.getD .anonymous ++ `_auto)
95+ let name ← name?.getDM (mkAuxDeclName `_auto)
9696 let type := Lean.mkConst `Lean.Syntax
9797 let value ← quoteAutoTactic tactic
9898 trace[Elab.autoParam] value
Original file line number Diff line number Diff line change @@ -15,7 +15,7 @@ example : U := by
1515
1616/--
1717trace: [ Meta.Tactic.simp.discharge ] bar discharge ✅️
18- autoParam T _auto✝
18+ autoParam T bar._auto_1
1919 [ Meta.Tactic.simp.rewrite ] T.mk:1000:
2020 T
2121 ==>
Original file line number Diff line number Diff line change @@ -29,7 +29,7 @@ def f (x := 0) (_ : x = x := by rfl) : Nat := x+1
2929
3030
3131/--
32- info: (x : optParam Nat 0) → autoParam (x = x) _auto✝ → Nat
32+ info: (x : optParam Nat 0) → autoParam (x = x) f._auto_1 → Nat
3333---
3434(x : Nat) → x = x → Nat
3535-/
You can’t perform that action at this time.
0 commit comments