@@ -22,7 +22,8 @@ namespace Lean.Elab.Tactic
2222open Lean Elab Parser Tactic Meta Simp Tactic.TryThis
2323
2424/-- Filter out `+suggestions` from the config syntax -/
25- def filterSuggestionsFromConfig (cfg : TSyntax ``Lean.Parser.Tactic.optConfig) : MetaM (TSyntax ``Lean.Parser.Tactic.optConfig) := do
25+ def filterSuggestionsFromSimpConfig (cfg : TSyntax ``Lean.Parser.Tactic.optConfig) :
26+ MetaM (TSyntax ``Lean.Parser.Tactic.optConfig) := do
2627 -- The config has one arg: a null node containing configItem nodes
2728 let nullNode := cfg.raw.getArg 0
2829 let configItems := nullNode.getArgs
@@ -67,7 +68,7 @@ def mkSimpCallStx (stx : Syntax) (usedSimps : UsedSimps) : MetaM (TSyntax `tacti
6768 else
6869 `(tactic| simp%$tk $cfg:optConfig $[$discharger]? $[only%$o]? [$argsArray,*] $[$loc]?)
6970 -- Build syntax for suggestion (without +suggestions config)
70- let filteredCfg ← filterSuggestionsFromConfig cfg
71+ let filteredCfg ← filterSuggestionsFromSimpConfig cfg
7172 let stxForSuggestion ← if bang.isSome then
7273 `(tactic| simp!%$tk $filteredCfg:optConfig $[$discharger]? $[only%$o]? [$argsArray,*] $[$loc]?)
7374 else
@@ -109,7 +110,7 @@ def mkSimpCallStx (stx : Syntax) (usedSimps : UsedSimps) : MetaM (TSyntax `tacti
109110 else
110111 `(tactic| simp_all%$tk $cfg:optConfig $[$discharger]? $[only%$o]? [$argsArray,*])
111112 -- Build syntax for suggestion (without +suggestions config)
112- let filteredCfg ← filterSuggestionsFromConfig cfg
113+ let filteredCfg ← filterSuggestionsFromSimpConfig cfg
113114 let stxForSuggestion ←
114115 if argsArray.isEmpty then
115116 if bang.isSome then
0 commit comments