comap
operation on mv_polynomial
#
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
This file defines the comap
function on mv_polynomial
.
mv_polynomial.comap
is a low-tech example of a map of "algebraic varieties," modulo the fact that
mathlib
does not yet define varieties.
Notation #
As in other polynomial files, we typically use the notation:
-
σ : Type*
(indexing the variables) -
R : Type*
[comm_semiring R]
(the coefficients)
Given an algebra hom f : mv_polynomial σ R →ₐ[R] mv_polynomial τ R
and a variable evaluation v : τ → R
,
comap f v
produces a variable evaluation σ → R
.
Equations
- mv_polynomial.comap f = λ (x : τ → R) (i : σ), ⇑(mv_polynomial.aeval x) (⇑f (mv_polynomial.X i))
If two polynomial types over the same coefficient ring R
are equivalent,
there is a bijection between the types of functions from their variable types to R
.
Equations
- mv_polynomial.comap_equiv f = {to_fun := mv_polynomial.comap ↑f, inv_fun := mv_polynomial.comap ↑(f.symm), left_inv := _, right_inv := _}