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 : Nat}
(hn : LT.lt 2 n)
{R : Type u_1}
[LinearOrderedCommRing R]
(x : R)
:
LT.lt 0 (eval x (cyclotomic n R))
theorem
Polynomial.cyclotomic_pos_and_nonneg
(n : Nat)
{R : Type u_1}
[LinearOrderedCommRing R]
(x : R)
:
And (LT.lt 1 x → LT.lt 0 (eval x (cyclotomic n R))) (LE.le 1 x → LE.le 0 (eval x (cyclotomic n R)))
theorem
Polynomial.cyclotomic_pos'
(n : Nat)
{R : Type u_1}
[LinearOrderedCommRing R]
{x : R}
(hx : LT.lt 1 x)
:
LT.lt 0 (eval x (cyclotomic n R))
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 : Nat)
{R : Type u_1}
[LinearOrderedCommRing R]
{x : R}
(hx : LE.le 1 x)
:
LE.le 0 (eval x (cyclotomic n R))
Cyclotomic polynomials are always nonnegative on inputs one or more.