Skip to content

Commit fa73f05

Browse files
committed
synthesizeSyntheticMVarsNoPostponing
1 parent e2dbabd commit fa73f05

File tree

5 files changed

+36
-7
lines changed

5 files changed

+36
-7
lines changed

REPL/Lean/InfoTree.lean

+3-6
Original file line numberDiff line numberDiff line change
@@ -200,12 +200,9 @@ Finds all appearances of `sorry` in an `InfoTree`, reporting
200200
-/
201201
def sorries (t : InfoTree) : List (ContextInfo × SorryType × Position × Position) :=
202202
(t.findSorryTacticNodes.map fun ⟨i, ctx⟩ =>
203-
if i.goalsBefore.isEmpty then
204-
dbgTrace "no goals at sorry!" fun _ => (ctx, panic "")
205-
else
206-
-- HACK: creating a child ngen
207-
({ ctx with mctx := i.mctxBefore, ngen := ctx.ngen.mkChild.1 }, .tactic i.goalsBefore.head!,
208-
stxRange ctx.fileMap i.stx)) ++
203+
-- HACK: creating a child ngen
204+
({ ctx with mctx := i.mctxBefore, ngen := ctx.ngen.mkChild.1 }, .tactic i.goalsBefore.head!,
205+
stxRange ctx.fileMap i.stx)) ++
209206
(t.findSorryTermNodes.map fun ⟨i, ctx⟩ =>
210207
(ctx, .term i.lctx i.expectedType?, stxRange ctx.fileMap i.stx))
211208

REPL/Snapshots.lean

+2-1
Original file line numberDiff line numberDiff line change
@@ -139,7 +139,8 @@ def runMetaM (p : ProofSnapshot) (t : MetaM α) : IO (α × ProofSnapshot) := do
139139

140140
/-- Run a `TermElabM` monadic function in the current `ProofSnapshot`, updating the `Term.State`. -/
141141
def runTermElabM (p : ProofSnapshot) (t : TermElabM α) : IO (α × ProofSnapshot) := do
142-
let ((a, termState), p') ← p.runMetaM (Lean.Elab.Term.TermElabM.run (s := p.termState) do t)
142+
let ((a, termState), p') ← p.runMetaM (Lean.Elab.Term.TermElabM.run (s := p.termState)
143+
(do let r ← t; Term.synthesizeSyntheticMVarsNoPostponing; pure r))
143144
return (a, { p' with termState })
144145

145146
/-- Run a `TacticM` monadic function in the current `ProofSnapshot`, updating the `Tactic.State`. -/
+22
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,22 @@
1+
{"env": 0}
2+
3+
{"sorries":
4+
[{"proofState": 0,
5+
"pos": {"line": 1, "column": 22},
6+
"goal": "⊢ False",
7+
"endPos": {"line": 1, "column": 27}}],
8+
"messages":
9+
[{"severity": "warning",
10+
"pos": {"line": 1, "column": 0},
11+
"endPos": {"line": 1, "column": 7},
12+
"data": "declaration uses 'sorry'"}],
13+
"env": 1}
14+
15+
{"proofState": 1,
16+
"messages":
17+
[{"severity": "error",
18+
"pos": {"line": 0, "column": 0},
19+
"endPos": {"line": 0, "column": 0},
20+
"data": "unsolved goals\n⊢ False"}],
21+
"goals": []}
22+

test/Mathlib/test/20240209.in

+5
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,5 @@
1+
{"cmd": "import Std.Tactic.Simpa"}
2+
3+
{"cmd": "example : False := by sorry", "env": 0}
4+
5+
{"tactic": "simpa using show False by done", "proofState": 0}

test/Mathlib/test/20240209.lean

+4
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,4 @@
1+
import Std.Tactic.Simpa
2+
3+
example : False := by
4+
simpa using show False by done

0 commit comments

Comments
 (0)