Cyclotomic polynomials and expand
. #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
We gather results relating cyclotomic polynomials and expand
.
Main results #
polynomial.cyclotomic_expand_eq_cyclotomic_mul
: Ifp
is a prime such that¬ p ∣ n
, thenexpand R p (cyclotomic n R) = (cyclotomic (n * p) R) * (cyclotomic n R)
.polynomial.cyclotomic_expand_eq_cyclotomic
: Ifp
is a prime such thatp ∣ n
, thenexpand R p (cyclotomic n R) = cyclotomic (p * n) R
.polynomial.cyclotomic_mul_prime_eq_pow_of_not_dvd
: IfR
is of characteristicp
and¬p ∣ n
, thencyclotomic (n * p) R = (cyclotomic n R) ^ (p - 1)
.polynomial.cyclotomic_mul_prime_dvd_eq_pow
: IfR
is of characteristicp
andp ∣ n
, thencyclotomic (n * p) R = (cyclotomic n R) ^ p
.polynomial.cyclotomic_mul_prime_pow_eq
: IfR
is of characteristicp
and¬p ∣ m
, thencyclotomic (p ^ k * m) R = (cyclotomic m R) ^ (p ^ k - p ^ (k - 1))
.polynomial.cyclotomic_mul_prime_pow_eq
: IfR
is of characteristicp
and¬p ∣ m
, thencyclotomic (p ^ k * m) R = (cyclotomic m R) ^ (p ^ k - p ^ (k - 1))
.
If p
is a prime such that ¬ p ∣ n
, then
expand R p (cyclotomic n R) = (cyclotomic (n * p) R) * (cyclotomic n R)
.
If p
is a prime such that p ∣ n
, then
expand R p (cyclotomic n R) = cyclotomic (p * n) R
.
If the p ^ n
th cyclotomic polynomial is irreducible, so is the p ^ m
th, for m ≤ n
.
If irreducible (cyclotomic (p ^ n) R)
then irreducible (cyclotomic p R).
If R
is of characteristic p
and ¬p ∣ n
, then
cyclotomic (n * p) R = (cyclotomic n R) ^ (p - 1)
.
If R
is of characteristic p
and p ∣ n
, then
cyclotomic (n * p) R = (cyclotomic n R) ^ p
.
If R
is of characteristic p
and ¬p ∣ m
, then ζ
is a root of cyclotomic (p ^ k * m) R
if and only if it is a primitive m
-th root of unity.