"Mirror" of a univariate polynomial #
In this file we define Polynomial.mirror
, a variant of Polynomial.reverse
. The difference
between reverse
and mirror
is that reverse
will decrease the degree if the polynomial is
divisible by X
.
Main definitions #
Main results #
Polynomial.mirror_mul_of_domain
:mirror
preserves multiplication.Polynomial.irreducible_of_mirror
: an irreducibility criterion involvingmirror
mirror of a polynomial: reverses the coefficients while preserving Polynomial.natDegree
Equations
- p.mirror = p.reverse * Polynomial.X ^ p.natTrailingDegree
Instances For
@[simp]
@[simp]
@[simp]
@[simp]
theorem
Polynomial.natDegree_mul_mirror
{R : Type u_1}
[Semiring R]
(p : Polynomial R)
[NoZeroDivisors R]
:
theorem
Polynomial.natTrailingDegree_mul_mirror
{R : Type u_1}
[Semiring R]
(p : Polynomial R)
[NoZeroDivisors R]
:
theorem
Polynomial.mirror_mul_of_domain
{R : Type u_1}
[Ring R]
(p q : Polynomial R)
[NoZeroDivisors R]
:
theorem
Polynomial.mirror_smul
{R : Type u_1}
[Ring R]
(p : Polynomial R)
[NoZeroDivisors R]
(a : R)
: