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 3a76a36 commit cb405b5Copy full SHA for cb405b5
src/Lean/Meta/Tactic/Grind/Split.lean
@@ -315,7 +315,8 @@ private def splitCore (c : SplitInfo) (numCases : Nat) (isRec : Bool) (stopAtFir
315
if let some falseProof ← getFalseProof? subgoal.mvarId then
316
goal.mvarId.assignFalseProof falseProof
317
return .closed seq
318
- else
+ else if !seq.isEmpty then
319
+ /- **Note**: if the sequence is empty, it means the user will never see this goal. -/
320
seqNew := seqNew.push seq
321
if (← goal.mvarId.getType).isFalse then
322
/- **Note**: We add the marker to assist `getFalseExpr?` -/
0 commit comments