Theory of univariate polynomials #
We prove basic results about univariate polynomials.
_ %ₘ q
as an R
-linear map.
Equations
- q.modByMonicHom = { toFun := fun (p : Polynomial R) => p %ₘ q, map_add' := ⋯, map_smul' := ⋯ }
Instances For
Equations
- ⋯ = ⋯
This lemma is useful for working with the intDegree
of a rational function.
Characterization of a unit of a polynomial ring over an integral domain R
.
See Polynomial.isUnit_iff_coeff_isUnit_isNilpotent
when R
is a commutative ring.
Alternate phrasing of Polynomial.Monic.irreducible_iff_natDegree'
where we only have to check
one divisor at a time.
Equations
- ⋯ = ⋯
McCoy theorem: a polynomial P : R[X]
is a zerodivisor if and only if there is a : R
such that a ≠ 0
and a • P = 0
.
The multiplicity of a
as root of a nonzero polynomial p
is at least n
iff
(X - a) ^ n
divides p
.
The multiplicity of a
as root of (X - a) ^ n
is n
.
The multiplicity of p + q
is at least the minimum of the multiplicities.
Division by a monic polynomial doesn't change the leading coefficient.
A polynomial over an integral domain R
is irreducible if it is monic and
irreducible after mapping into an integral domain S
.
A special case of this lemma is that a polynomial over ℤ
is irreducible if
it is monic and irreducible over ℤ/pℤ
for some prime p
.