Documentation

Mathlib.RingTheory.UniqueFactorizationDomain.Multiplicity

Unique factorization and multiplicity #

Main results #

theorem WfDvdMonoid.max_power_factor' {α : Type u_1} [CommMonoidWithZero α] [WfDvdMonoid α] {a₀ x : α} (h : a₀ 0) (hx : ¬IsUnit x) :
∃ (n : ) (a : α), ¬x a a₀ = x ^ n * a
theorem WfDvdMonoid.max_power_factor {α : Type u_1} [CommMonoidWithZero α] [WfDvdMonoid α] {a₀ x : α} (h : a₀ 0) (hx : Irreducible x) :
∃ (n : ) (a : α), ¬x a a₀ = x ^ n * a

The multiplicity of an irreducible factor of a nonzero element is exactly the number of times the normalized factor occurs in the normalizedFactors.

See also count_normalizedFactors_eq which expands the definition of multiplicity to produce a specification for count (normalizedFactors _) _..

The number of times an irreducible factor p appears in normalizedFactors x is defined by the number of times it divides x.

See also multiplicity_eq_count_normalizedFactors if n is given by multiplicity p x.

The number of times an irreducible factor p appears in normalizedFactors x is defined by the number of times it divides x. This is a slightly more general version of UniqueFactorizationMonoid.count_normalizedFactors_eq that allows p = 0.

See also multiplicity_eq_count_normalizedFactors if n is given by multiplicity p x.

@[deprecated WfDvdMonoid.max_power_factor]
theorem UniqueFactorizationMonoid.max_power_factor {R : Type u_2} [CancelCommMonoidWithZero R] [UniqueFactorizationMonoid R] {a₀ x : R} (h : a₀ 0) (hx : Irreducible x) :
∃ (n : ) (a : R), ¬x a a₀ = x ^ n * a

Deprecated. Use WfDvdMonoid.max_power_factor instead.