Equivalences between polynomial rings #
This file establishes a number of equivalences between polynomial rings, based on equivalences between the underlying types.
Notation #
As in other polynomial files, we typically use the notation:
-
σ : Type*
(indexing the variables) -
R : Type*
[CommSemiring R]
(the coefficients) -
s : σ →₀ ℕ
, a function fromσ
toℕ
which is zero away from a finite set. This will give rise to a monomial inMvPolynomial σ R
which mathematicians might callX^s
-
a : R
-
i : σ
, with corresponding monomialX i
, often denotedX_i
by mathematicians -
p : MvPolynomial σ R
Tags #
equivalence, isomorphism, morphism, ring hom, hom
The ring isomorphism between multivariable polynomials in a single variable and polynomials over the ground ring.
Instances For
If e : A ≃+* B
is an isomorphism of rings, then so is map e
.
Instances For
If e : A ≃ₐ[R] B
is an isomorphism of R
-algebras, then so is map e
.
Instances For
The function from multivariable polynomials in a sum of two types, to multivariable polynomials in one of the types, with coefficients in multivariable polynomials in the other type.
See sumRingEquiv
for the ring isomorphism.
Instances For
The function from multivariable polynomials in one type, with coefficients in multivariable polynomials in another type, to multivariable polynomials in the sum of the two types.
See sumRingEquiv
for the ring isomorphism.
Instances For
The algebra isomorphism between multivariable polynomials in no variables and the ground ring.
Instances For
The ring isomorphism between multivariable polynomials in no variables and the ground ring.
Instances For
A helper function for sumRingEquiv
.
Instances For
The ring isomorphism between multivariable polynomials in a sum of two types, and multivariable polynomials in one of the types, with coefficients in multivariable polynomials in the other type.
Instances For
The algebra isomorphism between multivariable polynomials in a sum of two types, and multivariable polynomials in one of the types, with coefficients in multivariable polynomials in the other type.
Instances For
The algebra isomorphism between multivariable polynomials in Option S₁
and
polynomials with coefficients in MvPolynomial S₁ R
.
Instances For
The algebra isomorphism between multivariable polynomials in Option S₁
and
multivariable polynomials with coefficients in polynomials.
Instances For
The algebra isomorphism between multivariable polynomials in Fin (n + 1)
and
polynomials over multivariable polynomials in Fin n
.
Instances For
The coefficient of m
in the i
-th coefficient of finSuccEquiv R n f
equals the
coefficient of Finsupp.cons i m
in f
.