Documentation

Mathlib.Algebra.Polynomial.Eval.Algebra

Evaluation of polynomials in an algebra #

This file concerns evaluating polynomials where the map is algebraMap

TODO: merge with parts of Algebra/Polynomial/AlgebraMap.lean?

@[simp]
theorem Polynomial.eval₂_mul' {R : Type u} {S : Type v} [CommSemiring R] [Semiring S] [Algebra R S] (x : S) (p q : Polynomial R) :
@[simp]
theorem Polynomial.eval₂_pow' {R : Type u} {S : Type v} [CommSemiring R] [Semiring S] [Algebra R S] (x : S) (p : Polynomial R) (n : ) :
@[simp]
theorem Polynomial.eval₂_comp' {R : Type u} {S : Type v} [CommSemiring R] [Semiring S] [Algebra R S] (x : S) (p q : Polynomial R) :