Documentation

Mathlib.RingTheory.UniqueFactorizationDomain.Finsupp

Factors as finsupp #

Main definitions #

noncomputable def factorization {α : Type u_1} [CommMonoidWithZero α] [UniqueFactorizationMonoid α] [NormalizationMonoid α] [DecidableEq α] (n : α) :

This returns the multiset of irreducible factors as a Finsupp.

Equations
Instances For
    @[simp]

    The support of factorization n is exactly the Finset of normalized factors

    @[simp]
    theorem factorization_mul {α : Type u_1} [CommMonoidWithZero α] [UniqueFactorizationMonoid α] [NormalizationMonoid α] [DecidableEq α] {a b : α} (ha : a 0) (hb : b 0) :

    For nonzero a and b, the power of p in a * b is the sum of the powers in a and b

    For any p, the power of p in x^n is n times the power in x