Lemmas related to Nat.Prime and lcm #
This file contains lemmas related to Nat.Prime.
These lemmas are kept separate from Mathlib/Data/Nat/GCD/Basic.lean in order to minimize imports.
Main results #
Nat.Prime.dvd_or_dvd_of_dvd_lcm: Ifp ∣ lcm a b, thenp ∣ a ∨ p ∣ b.Nat.Prime.dvd_lcm:p ∣ lcm a b ↔ p ∣ a ∨ p ∣ b.Nat.Prime.not_dvd_lcm: Ifp ∤ aandp ∤ b, thenp ∤ lcm a b.