Skip to content

Commit 82fea35

Browse files
committed
doc:
1 parent e94bc2d commit 82fea35

File tree

2 files changed

+2
-0
lines changed

2 files changed

+2
-0
lines changed

src/Lean/Elab/Tactic/Grind/Main.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -130,6 +130,7 @@ def mkGrindParams
130130
trace[grind.debug.inj] "{params.inj.getOrigins.map (·.pp)}"
131131
return params
132132

133+
-- **TODO**: Remove `Grind.Trace`
133134
def grind
134135
(mvarId : MVarId) (config : Grind.Config)
135136
(only : Bool)

src/Lean/Elab/Tactic/Try.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -378,6 +378,7 @@ where
378378
$tacs2*)
379379
modify (·.push tac)
380380

381+
-- **TODO**: Use `finish?` infrastructure
381382
private def evalSuggestGrindTrace : TryTactic := fun tac => do
382383
match tac with
383384
| `(tactic| grind? $configStx:optConfig $[only%$only]? $[ [$params:grindParam,*] ]?) =>

0 commit comments

Comments
 (0)