leanprover-community / mathlib

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

Zulip Chat Archive

Stream: Is there code for X?

Topic: Nat.exists_ne_zero


Kim Morrison (Jul 30 2024 at 03:58):

Do we have this somewhere?

@[simp] theorem Nat.exists_ne_zero {P : Nat → Prop} : (∃ n, ¬ n = 0 ∧ P n) ↔ ∃ n, P (n + 1) := ...

Yury G. Kudryashov (Jul 30 2024 at 04:06):

Probably, no.

Yaël Dillies (Jul 30 2024 at 06:20):

That's one application of the missing Nat.exists + simp afterwards


Last updated: May 02 2025 at 03:31 UTC

Theme Simple by wildflame © 2016 Powered by jekyll