Counit morphisms for multivariate polynomials #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
One may consider the ring of multivariate polynomials mv_polynomial A R
with coefficients in R
and variables indexed by A
. If A
is not just a type, but an algebra over R
,
then there is a natural surjective algebra homomorphism mv_polynomial A R →ₐ[R] A
obtained by X a ↦ a
.
Main declarations #
mv_polynomial.acounit R A
is the natural surjective algebra homomorphismmv_polynomial A R →ₐ[R] A
obtained byX a ↦ a
mv_polynomial.counit
is an “absolute” variant withR = ℤ
mv_polynomial.counit_nat
is an “absolute” variant withR = ℕ
mv_polynomial.acounit A B
is the natural surjective algebra homomorphism
mv_polynomial B A →ₐ[A] B
obtained by X a ↦ a
.
See mv_polynomial.counit
for the “absolute” variant with A = ℤ
,
and mv_polynomial.counit_nat
for the “absolute” variant with A = ℕ
.
Equations
mv_polynomial.counit R
is the natural surjective ring homomorphism
mv_polynomial R ℤ →+* R
obtained by X r ↦ r
.
See mv_polynomial.acounit
for a “relative” variant for algebras over a base ring,
and mv_polynomial.counit_nat
for the “absolute” variant with R = ℕ
.
Equations
mv_polynomial.counit_nat A
is the natural surjective ring homomorphism
mv_polynomial A ℕ →+* A
obtained by X a ↦ a
.
See mv_polynomial.acounit
for a “relative” variant for algebras over a base ring
and mv_polynomial.counit
for the “absolute” variant with A = ℤ
.