Factorization of monic poynomials of given degree #
This file contains two main results:
Polynomial.IsMonicOfDegree.eq_mul_isMonicOfDegree_one_isMonicOfDegree
shows that a monic polynomial of positive degree over an algebraically closed field can be written as a monic polynomial of degree 1 times another monic factor.Polynomial.IsMonicOfDegree.eq_mul_isMonicOfDegree_two_isMonicOfDegree
shows that a monic polynomial of degree at least two overℝ
can be written as a monic polynomial of degree two times another monic factor.
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
.