mathlib documentation

ring_theory.​euclidean_domain

ring_theory.​euclidean_domain

theorem span_gcd {α : Type u_1} [euclidean_domain α] (x y : α) :

theorem gcd_is_unit_iff {α : Type u_1} [euclidean_domain α] {x y : α} :

theorem is_coprime_of_dvd {α : Type u_1} [euclidean_domain α] {x y : α} :
¬(x = 0 y = 0)(∀ (z : α), z nonunits αz 0z x¬z y)is_coprime x y

theorem dvd_or_coprime {α : Type u_1} [euclidean_domain α] (x y : α) :