Skip to content

Commit 2a7c82c

Browse files
committed
chore: make auto param decls of private decls private
1 parent 455fd0b commit 2a7c82c

File tree

3 files changed

+3
-3
lines changed

3 files changed

+3
-3
lines changed

src/Lean/Elab/Binders.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -92,7 +92,7 @@ Returns the declaration name.
9292
-/
9393
def 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

tests/lean/run/3257.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -15,7 +15,7 @@ example : U := by
1515

1616
/--
1717
trace: [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
==>

tests/lean/run/cleanup_forallTelescope.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff 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
-/

0 commit comments

Comments
 (0)