Documentation

Mathlib.Analysis.Polynomial.Factorization

Factorization of monic poynomials of given degree #

This file contains two main results:

theorem Polynomial.IsMonicOfDegree.eq_isMonicOfDegree_one_mul_isMonicOfDegree {F : Type u_1} [Field F] [IsAlgClosed F] {f : Polynomial F} {n : } (hf : f.IsMonicOfDegree (n + 1)) :
∃ (f₁ : Polynomial F) (f₂ : Polynomial F), f₁.IsMonicOfDegree 1 f₂.IsMonicOfDegree n f = f₁ * f₂

If f : F[X] is monic of degree ≥ 1 and F is an algebraically closed field, then f = f₁ * f₂ with f₁ monic of degree 1 and f₂ monic of degree f.natDegree - 1.

If f : ℝ[X] is monic of positive degree, then f = f₁ * f₂ with f₁ monic of degree 1 or 2.

This relies on the fact that irreducible polynomials over have degree at most 2.

If f : ℝ[X] is monic of degree ≥ 2, then f = f₁ * f₂ with f₁ monic of degree 2 and f₂ monic of degree f.natDegree - 2.

This relies on the fact that irreducible polynomials over have degree at most 2.