We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
1 parent b1793a3 commit 2012f87Copy full SHA for 2012f87
Mathlib/Tactic/TacticAnalysis/Declarations.lean
@@ -360,7 +360,7 @@ register_option linter.tacticAnalysis.tryAtEachStepSimpAllSuggestions : Bool :=
360
361
@[tacticAnalysis linter.tacticAnalysis.tryAtEachStepSimpAllSuggestions,
362
inherit_doc linter.tacticAnalysis.tryAtEachStepSimpAllSuggestions]
363
-def tryAtEachStepSimpAllSuggestions := tryAtEachStep fun _ _ => `(tactic| try simp_all? +suggestions)
+def tryAtEachStepSimpAllSuggestions := tryAtEachStep fun _ _ => `(tactic| simp_all? +suggestions)
364
365
-- /-- Run `canonical +suggestions` at every step in proofs, reporting where it succeeds. -/
366
-- register_option linter.tacticAnalysis.tryAtEachStepCanonicalSuggestions : Bool := {
0 commit comments