Documentation

Mathlib.FieldTheory.IsAlgClosed.Classification

Classification of Algebraically closed fields #

This file contains results related to classifying algebraically closed fields.

Main statements #

The cardinality of an algebraic extension is at most the maximum of the cardinality of the base ring or ℵ₀

theorem IsAlgClosed.isAlgClosure_of_transcendence_basis {R : Type u_1} {K : Type u_3} [CommRing R] [Field K] [Algebra R K] {ι : Type u_4} (v : ιK) [IsAlgClosed K] (hv : IsTranscendenceBasis R v) :
def IsAlgClosed.equivOfTranscendenceBasis {R : Type u_1} {L : Type u_2} {K : Type u_3} [CommRing R] [Field K] [Algebra R K] [Field L] [Algebra R L] {ι : Type u_4} (v : ιK) {κ : Type u_5} (w : κL) [IsAlgClosed K] [IsAlgClosed L] (e : ι κ) (hv : IsTranscendenceBasis R v) (hw : IsTranscendenceBasis R w) :
K ≃+* L

setting R to be ZMod (ringChar R) this result shows that if two algebraically closed fields have equipotent transcendence bases and the same characteristic then they are isomorphic.

Equations
  • One or more equations did not get rendered due to their size.
Instances For

    If K is an uncountable algebraically closed field, then its cardinality is the same as that of a transcendence basis.

    Two uncountable algebraically closed fields of characteristic zero are isomorphic if they have the same cardinality.

    Two uncountable algebraically closed fields are isomorphic if they have the same cardinality and the same characteristic.