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.
searchUsing
1 parent 5e3c330 commit 41458a0Copy full SHA for 41458a0
src/Lean/Meta/Tactic/Grind/SearchM.lean
@@ -219,4 +219,14 @@ def nextGoal? : SearchM (Option Nat) := do
219
return some choice.generation
220
unreachable!
221
222
+/--
223
+Execute `x` using the current goal as the starting goal.
224
+The state is not updated.
225
+-/
226
+def searchUsing (x : SearchM α) : GoalM α := do
227
+ let goal ← get
228
+ let goal := { goal with newFacts := {} }
229
+ let (a, _) ← x.run goal
230
+ return a
231
+
232
end Lean.Meta.Grind
0 commit comments