leanprover-community / mathlib

  • Home
  • Zulip archive
  • API documentation
  • Lean web editor
  • Links

Zulip Chat Archive

Stream: Is there code for X?

Topic: sub one succ


Bolton Bailey (Aug 10 2022 at 23:09):

I'm looking for this lemma, is it in mathlib?

lemma nat.sub_one_succ (n : ℕ) (h : 0 < n) : nat.succ (n-1) = n :=
begin
  library_search,
end

Eric Rodriguez (Aug 10 2022 at 23:13):

docs#nat.succ_pred_eq_of_pos


Last updated: May 02 2025 at 03:31 UTC

Theme Simple by wildflame © 2016 Powered by jekyll