Skip to content

Commit

Permalink
fix: patch for std4#193 (#6188)
Browse files Browse the repository at this point in the history
fix: patch for std4#193
  • Loading branch information
fgdorais committed Aug 17, 2023
1 parent ae74c2e commit 5f5c4e1
Show file tree
Hide file tree
Showing 2 changed files with 1 addition and 10 deletions.
9 changes: 0 additions & 9 deletions Mathlib/Init/Data/Nat/Lemmas.lean
Original file line number Diff line number Diff line change
Expand Up @@ -500,15 +500,6 @@ def subInduction {P : ℕ → ℕ → Sort u} (H1 : ∀ m, P 0 m) (H2 : ∀ n, P
| succ n, succ m => H3 _ _ (subInduction H1 H2 H3 n m)
#align nat.sub_induction Nat.subInduction

protected def strongRecOn {p : Nat → Sort u} (n : Nat) (h : ∀ n, (∀ m, m < n → p m) → p n) :
p n := by
suffices ∀ n m, m < n → p m from this (succ n) n (lt_succ_self _)
intro n; induction' n with n ih
· intro m h₁; exact absurd h₁ m.not_lt_zero
· intro m h₁
apply Or.by_cases (Decidable.lt_or_eq_of_le (le_of_lt_succ h₁))
· intros; apply ih; assumption
· intros; subst m; apply h _ ih
#align nat.strong_rec_on Nat.strongRecOn

-- porting note: added `elab_as_elim`
Expand Down
2 changes: 1 addition & 1 deletion lake-manifest.json
Original file line number Diff line number Diff line change
Expand Up @@ -28,6 +28,6 @@
{"git":
{"url": "https://github.com/leanprover/std4",
"subDir?": null,
"rev": "dbffa8cb31b0c51b151453c4ff8f00ede2a84ed8",
"rev": "8b864260672b21d964d79ecb2376e01d0eab9f5b",
"name": "std",
"inputRev?": "main"}}]}

0 comments on commit 5f5c4e1

Please sign in to comment.