Universal factorization ring #
Let R be a commutative ring and p : R[X] be monic of degree n and let n = m + k.
We construct the universal ring of the following functors on R-Alg:
S ↦ "monic polynomials over S of degree n": Represented byR[X₁,...,Xₙ]. SeeMvPolynomial.mapEquivMonic.S ↦ "factorizations of p into (monic deg m) * (monic deg k) in S": Represented by anR-algebra (Polynomial.UniversalFactorizationRing) that is finitely-presented as anR-module. SeePolynomial.UniversalFactorizationRing.homEquiv.S ↦ "factorizations of p into coprime (monic deg m) * (monic deg k) in S": Represented by an etaleR-algebra (TODO).
The free monic polynomial of degree n, as a polynomial in R[X₁,...,Xₙ][X].
Equations
- Polynomial.freeMonic R n = Polynomial.X ^ n + ∑ i : Fin n, Polynomial.C (MvPolynomial.X i) * Polynomial.X ^ ↑i
Instances For
The free monic polynomial of degree n, as a MonicDegreeEq in R[X₁,...,Xₙ][X].
Equations
Instances For
In light of the fact that MonicDegreeEq · n is representable by R[X₁,...,Xₙ],
this is the map R[X₁,...,Xₘ₊ₖ] → R[X₁,...,Xₘ] ⊗ R[X₁,...,Xₖ] corresponding to the multiplication
MonicDegreeEq · m × MonicDegreeEq · k → MonicDegreeEq · (m + k).
Equations
- One or more equations did not get rendered due to their size.
Instances For
Lifts along universalFactorizationMap corresponds to factorization of p into
monic polynomials with fixed degrees.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The canonical presentation of universalFactorizationMap.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The universal factorization ring of a monic polynomial p of degree n.
This is the representing object of the functor
S ↦ "factorizations of p into (monic deg m) * (monic deg k) in S".
See UniversalFactorizationRing.homEquiv.
Equations
- Polynomial.UniversalFactorizationRing m k hn p = TensorProduct (MvPolynomial (Fin n) R) R (TensorProduct R (MvPolynomial (Fin m) R) (MvPolynomial (Fin k) R))
Instances For
The canonical map R[X₁,...,Xₘ] ⊗ R[X₁,...,Xₙ] → UniversalFactorizationRing.
Equations
Instances For
The image of p in the universal factorization ring of p.
Equations
- Polynomial.UniversalFactorizationRing.monicDegreeEq m k hn p = ⟨Polynomial.map (algebraMap R (Polynomial.UniversalFactorizationRing m k hn p)) ↑p, ⋯⟩
Instances For
The first factor of p in the universal factorization ring of p.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The second factor of p in the universal factorization ring of p.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The universal factorization ring that represents
S ↦ "factorizations of p into (monic deg m) * (monic deg k) in S".
Equations
- One or more equations did not get rendered due to their size.