leanprover-community / mathlib

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

Zulip Chat Archive

Stream: Is there code for X?

Topic: equivalent formulation of "is not divisible"


Floris van Doorn (Oct 06 2020 at 02:45):

Is this in mathlib? I need the direction from right to left.

lemma not_dvd_iff (n m : ℕ) : ¬ n ∣ m ↔ ∃ k, n * k < m ∧ m < n * (k + 1)

Johan Commelin (Oct 06 2020 at 03:04):

I don't recognise it


Last updated: May 02 2025 at 03:31 UTC

Theme Simple by wildflame © 2016 Powered by jekyll