Algebraic Independence #
This file defines algebraic independence of a family of element of an R
algebra.
Main definitions #
AlgebraicIndependent
-AlgebraicIndependent R x
states the family of elementsx
is algebraically independent overR
, meaning that the canonical map out of the multivariable polynomial ring is injective.AlgebraicIndependent.aevalEquiv
- The canonical isomorphism from the polynomial ring to the subalgebra generated by an algebraic independent family.AlgebraicIndependent.repr
- The canonical map from the subalgebra generated by an algebraic independent family into the polynomial ring. It is the inverse ofAlgebraicIndependent.aevalEquiv
.AlgebraicIndependent.aevalEquivField
- The canonical isomorphism from the rational function field ring to the intermediate field generated by an algebraic independent family.AlgebraicIndependent.reprField
- The canonical map from the intermediate field generated by an algebraic independent family into the rational function field. It is the inverse ofAlgebraicIndependent.aevalEquivField
.IsTranscendenceBasis R x
- a familyx
is a transcendence basis overR
if it is a maximal algebraically independent subset.
References #
TODO #
Define the transcendence degree and show it is independent of the choice of a transcendence basis.
Tags #
transcendence basis, transcendence degree, transcendence
AlgebraicIndependent R x
states the family of elements x
is algebraically independent over R
, meaning that the canonical
map out of the multivariable polynomial ring is injective.
Equations
Instances For
A one-element family x
is algebraically independent if and only if
its element is transcendental.
The one-element family ![x]
is algebraically independent if and only if
x
is transcendental.
If a family x
is algebraically independent, then any of its element is transcendental.
If x = {x_i : A | i : ι}
and f = {f_i : MvPolynomial ι R | i : ι}
are algebraically
independent over R
, then {f_i(x) | i : ι}
is also algebraically independent over R
.
For the partial converse, see AlgebraicIndependent.of_aeval
.
If {f_i(x) | i : ι}
is algebraically independent over R
, then
{f_i : MvPolynomial ι R | i : ι}
is also algebraically independent over R
.
In fact, the x = {x_i : A | i : ι}
is also transcendental over R
provided that R
is a field and ι
is finite; the proof needs transcendence degree.
If A/R
is algebraic, then all algebraically independent families are empty.
Alias of the forward direction of algebraicIndependent_subtype_range
.
A set of algebraically independent elements in an algebra A
over a ring K
is also
algebraically independent over a subring R
of K
.
Every finite subset of an algebraically independent set is algebraically independent.
If every finite set of algebraically independent element has cardinality at most n
,
then the same is true for arbitrary sets of algebraically independent elements.
Canonical isomorphism between polynomials and the subalgebra generated by algebraically independent elements.
Equations
- hx.aevalEquiv = (AlgEquiv.ofInjective (MvPolynomial.aeval x) ⋯).trans ((MvPolynomial.aeval x).range.equivOfEq (Algebra.adjoin R (Set.range x)) ⋯)
Instances For
The canonical map from the subalgebra generated by an algebraic independent family into the polynomial ring.
Equations
- hx.repr = ↑hx.aevalEquiv.symm
Instances For
Canonical isomorphism between rational function field and the intermediate field generated by algebraically independent elements.
Equations
- hx.aevalEquivField = (let_fun this := AlgEquiv.ofInjectiveField (IsFractionRing.liftAlgHom ⋯); this).trans (IntermediateField.equivOfEq ⋯)
Instances For
The canonical map from the intermediate field generated by an algebraic independent family into the rational function field.
Equations
- hx.reprField = ↑hx.aevalEquivField.symm
Instances For
The isomorphism between MvPolynomial (Option ι) R
and the polynomial ring over
the algebra generated by an algebraically independent family.
Equations
- hx.mvPolynomialOptionEquivPolynomialAdjoin = (MvPolynomial.optionEquivLeft R ι).toRingEquiv.trans (Polynomial.mapEquiv hx.aevalEquiv.toRingEquiv)
Instances For
simp
-normal form of mvPolynomialOptionEquivPolynomialAdjoin_C
Variant of algebraicIndependent_of_finite
using Transcendental
.
Type
version of algebraicIndependent_of_finite'
.
If for each i : ι
, f_i : R[X]
is transcendental over R
, then {f_i(X_i) | i : ι}
in MvPolynomial ι R
is algebraically independent over R
.
If {x_i : A | i : ι}
is algebraically independent over R
, and for each i
,
f_i : R[X]
is transcendental over R
, then {f_i(x_i) | i : ι}
is also
algebraically independent over R
.
A family is a transcendence basis if it is a maximal algebraically independent subset.
Equations
- IsTranscendenceBasis R x = (AlgebraicIndependent R x ∧ ∀ (s : Set A), AlgebraicIndependent R Subtype.val → Set.range x ≤ s → Set.range x = s)
Instances For
Type
version of exists_isTranscendenceBasis
.
If x
is a transcendence basis of A/R
, then it is empty if and only if
A/R
is algebraic.
If x
is a transcendence basis of A/R
, then it is not empty if and only if
A/R
is transcendental.