Documentation

Mathlib.Data.Nat.GCD.Prime

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 #

theorem Nat.Prime.dvd_or_dvd_of_dvd_lcm {p a b : } (hp : Prime p) (h : p a.lcm b) :
p a p b
theorem Nat.Prime.dvd_lcm {p a b : } (hp : Prime p) :
p a.lcm b p a p b
theorem Nat.Prime.not_dvd_lcm {p a b : } (hp : Prime p) (ha : ¬p a) (hb : ¬p b) :
¬p a.lcm b