Documentation

Mathlib.Algebra.Polynomial.Mirror

"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 #

noncomputable def Polynomial.mirror {R : Type u_1} [Semiring R] (p : Polynomial R) :

mirror of a polynomial: reverses the coefficients while preserving Polynomial.natDegree

Equations
Instances For
    @[simp]
    theorem Polynomial.mirror_C {R : Type u_1} [Semiring R] (a : R) :
    Polynomial.mirror (Polynomial.C a) = Polynomial.C a
    theorem Polynomial.mirror_X {R : Type u_1} [Semiring R] :
    Polynomial.mirror Polynomial.X = Polynomial.X
    theorem Polynomial.mirror_involutive {R : Type u_1} [Semiring R] :
    Function.Involutive Polynomial.mirror
    @[simp]
    theorem Polynomial.mirror_eq_zero {R : Type u_1} [Semiring R] {p : Polynomial R} :