Skip to content

Commit 28b816b

Browse files
committed
unused argument linter
1 parent 11f7727 commit 28b816b

File tree

1 file changed

+1
-1
lines changed

1 file changed

+1
-1
lines changed

Mathlib/Data/Nat/Order/Basic.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -323,7 +323,7 @@ theorem diag_induction (P : ℕ → ℕ → Prop) (ha : ∀ a, P (a + 1) (a + 1)
323323
have _ : a + (b + 1) < (a + 1) + (b + 1) := by simp
324324
apply diag_induction P ha hb hd a (b + 1)
325325
apply lt_of_le_of_lt (Nat.le_succ _) h
326-
termination_by a b c => a + b
326+
termination_by a b => a + b
327327
decreasing_by all_goals assumption
328328
#align nat.diag_induction Nat.diag_induction
329329

0 commit comments

Comments
 (0)