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 e94bc2d commit 82fea35Copy full SHA for 82fea35
src/Lean/Elab/Tactic/Grind/Main.lean
@@ -130,6 +130,7 @@ def mkGrindParams
130
trace[grind.debug.inj] "{params.inj.getOrigins.map (·.pp)}"
131
return params
132
133
+-- **TODO**: Remove `Grind.Trace`
134
def grind
135
(mvarId : MVarId) (config : Grind.Config)
136
(only : Bool)
src/Lean/Elab/Tactic/Try.lean
@@ -378,6 +378,7 @@ where
378
$tacs2*)
379
modify (·.push tac)
380
381
+-- **TODO**: Use `finish?` infrastructure
382
private def evalSuggestGrindTrace : TryTactic := fun tac => do
383
match tac with
384
| `(tactic| grind? $configStx:optConfig $[only%$only]? $[ [$params:grindParam,*] ]?) =>
0 commit comments