Documentation

Mathlib.RingTheory.Polynomial.GaussLemma

Gauss's Lemma #

Gauss's Lemma is one of a few results pertaining to irreducibility of primitive polynomials.

Main Results #

theorem integralClosure.mem_lifts_of_monic_of_dvd_map {R : Type u_1} [CommRing R] (K : Type u_2) [Field K] [Algebra R K] {f : Polynomial R} (hf : f.Monic) {g : Polynomial K} (hg : g.Monic) (hd : Dvd.dvd g (Polynomial.map (algebraMap R K) f)) :

If K = Frac(R) and g : K[X] divides a monic polynomial with coefficients in R, then g * (C g.leadingCoeff⁻¹) has coefficients in R

theorem Polynomial.IsPrimitive.isUnit_iff_isUnit_map {R : Type u_1} [CommRing R] {K : Type u_2} [Field K] [Algebra R K] [IsFractionRing R K] {p : Polynomial R} (hp : p.IsPrimitive) :
Iff (IsUnit p) (IsUnit (map (algebraMap R K) p))

Gauss's Lemma for integrally closed domains states that a monic polynomial is irreducible iff it is irreducible in the fraction field.

theorem Polynomial.isIntegrallyClosed_iff' {R : Type u_1} [CommRing R] {K : Type u_2} [Field K] [Algebra R K] [IsFractionRing R K] [IsDomain R] :

Integrally closed domains are precisely the domains for in which Gauss's lemma holds for monic polynomials

Gauss's Lemma for GCD domains states that a primitive polynomial is irreducible iff it is irreducible in the fraction field.

Gauss's Lemma for states that a primitive integer polynomial is irreducible iff it is irreducible over .