Evaluating cyclotomic polynomials #
This file states some results about evaluating cyclotomic polynomials in various different ways.
Main definitions #
Polynomial.eval(₂)_one_cyclotomic_prime(_pow)
:eval 1 (cyclotomic p^k R) = p
.Polynomial.eval_one_cyclotomic_not_prime_pow
: Otherwise,eval 1 (cyclotomic n R) = 1
.Polynomial.cyclotomic_pos
:∀ x, 0 < eval x (cyclotomic n R)
if2 < n
.
theorem
Polynomial.cyclotomic_pos
{n : ℕ}
(hn : 2 < n)
{R : Type u_1}
[LinearOrderedCommRing R]
(x : R)
:
theorem
Polynomial.cyclotomic_pos_and_nonneg
(n : ℕ)
{R : Type u_1}
[LinearOrderedCommRing R]
(x : R)
:
theorem
Polynomial.cyclotomic_pos'
(n : ℕ)
{R : Type u_1}
[LinearOrderedCommRing R]
{x : R}
(hx : 1 < x)
:
Cyclotomic polynomials are always positive on inputs larger than one.
Similar to cyclotomic_pos
but with the condition on the input rather than index of the
cyclotomic polynomial.
theorem
Polynomial.cyclotomic_nonneg
(n : ℕ)
{R : Type u_1}
[LinearOrderedCommRing R]
{x : R}
(hx : 1 ≤ x)
:
Cyclotomic polynomials are always nonnegative on inputs one or more.