Skip to content

Commit

Permalink
chore(RingTheory): split AlgebraicIndependent.lean
Browse files Browse the repository at this point in the history
As a follow-up to splitting `RingTheory/Algebraic.lean`, also split `AlgebraicIndependent.lean`.

This PR creates the following new files:
* `AlgebraicIndependent/Defs.lean`: definition of `AlgebraicIndependent` and `IsTranscendenceBasis`
* `AlgebraicIndependent/Basic.lean`: basic results on `AlgebraicIndependent`
* `AlgebraicIndependent/TranscendenceBasis.lean`: basic results on `TranscendenceBasis`
* `AlgebraicIndependent/Adjoin.lean`: relating `AlgebraicIndependent` and `IntermediateField.adjoin`
* `AlgebraicIndependent/Transcendental.lean`: relating `AlgebraicIndependent`, `Transcendental` and `Algebraic`
* `AlgebraicIndependent/RankAndCardinality.lean`: about the rank/cardinality of `TranscendenceBasis`es
  • Loading branch information
Vierkantor committed Dec 2, 2024
1 parent 675c28e commit e1183fc
Show file tree
Hide file tree
Showing 10 changed files with 1,049 additions and 808 deletions.
7 changes: 6 additions & 1 deletion Mathlib.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4226,7 +4226,12 @@ import Mathlib.RingTheory.Algebraic.Integral
import Mathlib.RingTheory.Algebraic.LinearIndependent
import Mathlib.RingTheory.Algebraic.MvPolynomial
import Mathlib.RingTheory.Algebraic.Pi
import Mathlib.RingTheory.AlgebraicIndependent
import Mathlib.RingTheory.AlgebraicIndependent.Adjoin
import Mathlib.RingTheory.AlgebraicIndependent.Basic
import Mathlib.RingTheory.AlgebraicIndependent.Defs
import Mathlib.RingTheory.AlgebraicIndependent.RankAndCardinality
import Mathlib.RingTheory.AlgebraicIndependent.TranscendenceBasis
import Mathlib.RingTheory.AlgebraicIndependent.Transcendental
import Mathlib.RingTheory.Artinian
import Mathlib.RingTheory.Bezout
import Mathlib.RingTheory.Bialgebra.Basic
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/FieldTheory/IsAlgClosed/Classification.lean
Original file line number Diff line number Diff line change
Expand Up @@ -8,7 +8,7 @@ import Mathlib.Algebra.MvPolynomial.Cardinal
import Mathlib.Algebra.Polynomial.Cardinal
import Mathlib.FieldTheory.IsAlgClosed.Basic
import Mathlib.RingTheory.Algebraic.Cardinality
import Mathlib.RingTheory.AlgebraicIndependent
import Mathlib.RingTheory.AlgebraicIndependent.TranscendenceBasis

/-!
# Classification of Algebraically closed fields
Expand Down
3 changes: 2 additions & 1 deletion Mathlib/FieldTheory/SeparableDegree.lean
Original file line number Diff line number Diff line change
Expand Up @@ -7,7 +7,8 @@ import Mathlib.FieldTheory.SplittingField.Construction
import Mathlib.FieldTheory.IsAlgClosed.AlgebraicClosure
import Mathlib.FieldTheory.Separable
import Mathlib.FieldTheory.NormalClosure
import Mathlib.RingTheory.AlgebraicIndependent
import Mathlib.RingTheory.AlgebraicIndependent.Adjoin
import Mathlib.RingTheory.AlgebraicIndependent.TranscendenceBasis
import Mathlib.RingTheory.Polynomial.SeparableDegree
import Mathlib.RingTheory.Polynomial.UniqueFactorization

Expand Down
Loading

0 comments on commit e1183fc

Please sign in to comment.