Skip to content

Commit 1eff493

Browse files
committed
fix native_decide
1 parent 9caad98 commit 1eff493

File tree

1 file changed

+1
-1
lines changed

1 file changed

+1
-1
lines changed

src/Lean/Elab/Tactic/ElabTerm.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -416,7 +416,7 @@ private unsafe def elabNativeDecideCoreUnsafe (tacticName : Name) (expectedType
416416
-- disable async codegen so we can catch its exceptions; we don't want to report `evalConst`
417417
-- failures below when the actual reason was a codegen failure
418418
withOptions (Elab.async.set · false) do
419-
addAndCompile decl
419+
addAndCompile (mayPostPoneCompile := false) decl
420420
catch ex =>
421421
throwError m!"Tactic `{tacticName}` failed. Error: {ex.toMessageData}"
422422

0 commit comments

Comments
 (0)