Skip to content

Commit 2f07b70

Browse files
authored
fix: default parameter value in constructor footgun at cases tactic (#10939)
This PR fixes another instance of the “default parameter value in constructor” footgun, which was affecting the `cases` tactic in the `grind` interactive mode.
1 parent 09b36c3 commit 2f07b70

File tree

2 files changed

+5
-5
lines changed

2 files changed

+5
-5
lines changed

src/Lean/Meta/Tactic/Grind/Split.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -503,7 +503,7 @@ Tries to perform a case-split using `c`. Returns `none` if `c` has already been
503503
is not ready.
504504
-/
505505
def split? (c : SplitInfo) : SearchM (Option (List Goal × Nat)) := do
506-
let .ready numCases isRec ← checkSplitStatus c | return none
506+
let .ready numCases isRec _ ← checkSplitStatus c | return none
507507
let mvarId := (← getGoal).mvarId
508508
return some (← splitCore mvarId c numCases isRec)
509509

tests/lean/run/grind_ite_trace.lean

Lines changed: 4 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -93,8 +93,8 @@ theorem normalize_spec (assign : Std.HashMap Nat Bool) (e : IfExpr) :
9393
next => grind => finish?
9494
next => grind => finish?
9595
next => grind => finish?
96-
next => grind => finish -- TODO: ensure `finish?` works here
97-
next => grind => finish -- TODO: ensure `finish?` works here
96+
next => grind => finish?
97+
next => grind => finish?
9898
next => grind => finish?
9999

100100
example (assign : Std.HashMap Nat Bool) (e : IfExpr) :
@@ -108,6 +108,6 @@ example (assign : Std.HashMap Nat Bool) (e : IfExpr) :
108108
next => grind => finish?
109109
next => grind => finish?
110110
next => grind => finish?
111-
next => grind => finish -- TODO: ensure `finish?` works here
112-
next => grind => finish -- TODO: ensure `finish?` works here
111+
next => grind => finish?
112+
next => grind => finish?
113113
next => grind => finish?

0 commit comments

Comments
 (0)