Documentation

Mathlib.FieldTheory.Galois

Galois Extensions #

In this file we define Galois extensions as extensions which are both separable and normal.

Main definitions #

Main results #

Together, these two results prove the Galois correspondence.

class IsGalois (F : Type u_1) [Field F] (E : Type u_2) [Field E] [Algebra F E] :

A field extension E/F is Galois if it is both separable and normal. Note that in mathlib a separable extension of fields is by definition algebraic.

Instances
    theorem isGalois_iff {F : Type u_1} [Field F] {E : Type u_2} [Field E] [Algebra F E] :
    theorem IsGalois.integral (F : Type u_1) [Field F] {E : Type u_2} [Field E] [Algebra F E] [IsGalois F E] (x : E) :
    theorem IsGalois.separable (F : Type u_1) [Field F] {E : Type u_2} [Field E] [Algebra F E] [IsGalois F E] (x : E) :
    theorem IsGalois.splits (F : Type u_1) [Field F] {E : Type u_2} [Field E] [Algebra F E] [IsGalois F E] (x : E) :
    theorem IsGalois.IntermediateField.AdjoinSimple.card_aut_eq_finrank (F : Type u_1) [Field F] (E : Type u_2) [Field E] [Algebra F E] [FiniteDimensional F E] {α : E} (hα : IsIntegral F α) (h_sep : Polynomial.Separable (minpoly F α)) (h_splits : Polynomial.Splits (algebraMap F { x // x Fα }) (minpoly F α)) :
    Fintype.card ({ x // x Fα } ≃ₐ[F] { x // x Fα }) = FiniteDimensional.finrank F { x // x Fα }
    theorem IsGalois.tower_top_of_isGalois (F : Type u_1) (K : Type u_2) (E : Type u_3) [Field F] [Field K] [Field E] [Algebra F K] [Algebra F E] [Algebra K E] [IsScalarTower F K E] [IsGalois F E] :
    theorem isGalois_iff_isGalois_bot {F : Type u_1} {E : Type u_3} [Field F] [Field E] [Algebra F E] :
    IsGalois { x // x } E IsGalois F E
    theorem IsGalois.of_algEquiv {F : Type u_1} {E : Type u_3} [Field F] [Field E] {E' : Type u_4} [Field E'] [Algebra F E'] [Algebra F E] [IsGalois F E] (f : E ≃ₐ[F] E') :
    theorem AlgEquiv.transfer_galois {F : Type u_1} {E : Type u_3} [Field F] [Field E] {E' : Type u_4} [Field E'] [Algebra F E'] [Algebra F E] (f : E ≃ₐ[F] E') :
    theorem isGalois_iff_isGalois_top {F : Type u_1} {E : Type u_3} [Field F] [Field E] [Algebra F E] :
    IsGalois F { x // x } IsGalois F E
    instance isGalois_bot {F : Type u_1} {E : Type u_3} [Field F] [Field E] [Algebra F E] :
    IsGalois F { x // x }
    Equations
    def FixedPoints.intermediateField {F : Type u_1} [Field F] {E : Type u_2} [Field E] [Algebra F E] (M : Type u_3) [Monoid M] [MulSemiringAction M E] [SMulCommClass M F E] :

    The intermediate field of fixed points fixed by a monoid action that commutes with the F-action on E.

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      def IntermediateField.fixedField {F : Type u_1} [Field F] {E : Type u_2} [Field E] [Algebra F E] (H : Subgroup (E ≃ₐ[F] E)) :

      The intermediate field fixed by a subgroup

      Equations
      Instances For
        def IntermediateField.fixingSubgroup {F : Type u_1} [Field F] {E : Type u_2} [Field E] [Algebra F E] (K : IntermediateField F E) :

        The subgroup fixing an intermediate field

        Equations
        Instances For
          def IntermediateField.fixingSubgroupEquiv {F : Type u_1} [Field F] {E : Type u_2} [Field E] [Algebra F E] (K : IntermediateField F E) :

          The fixing subgroup of K : IntermediateField F E is isomorphic to E ≃ₐ[K] E

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

            The Galois correspondence from intermediate fields to subgroups

            Equations
            • One or more equations did not get rendered due to their size.
            Instances For
              def IsGalois.galoisInsertionIntermediateFieldSubgroup {F : Type u_1} [Field F] {E : Type u_2} [Field E] [Algebra F E] [FiniteDimensional F E] :
              GaloisInsertion (OrderDual.toDual IntermediateField.fixingSubgroup) (IntermediateField.fixedField OrderDual.toDual)

              The Galois correspondence as a GaloisInsertion

              Equations
              • One or more equations did not get rendered due to their size.
              Instances For
                def IsGalois.galoisCoinsertionIntermediateFieldSubgroup {F : Type u_1} [Field F] {E : Type u_2} [Field E] [Algebra F E] [FiniteDimensional F E] [IsGalois F E] :
                GaloisCoinsertion (OrderDual.toDual IntermediateField.fixingSubgroup) (IntermediateField.fixedField OrderDual.toDual)

                The Galois correspondence as a GaloisCoinsertion

                Equations
                • One or more equations did not get rendered due to their size.
                Instances For
                  theorem IsGalois.of_separable_splitting_field_aux {F : Type u_1} [Field F] {E : Type u_2} [Field E] [Algebra F E] {p : Polynomial F} [hFE : FiniteDimensional F E] [sp : Polynomial.IsSplittingField F E p] (hp : Polynomial.Separable p) (K : Type u_3) [Field K] [Algebra F K] [Algebra K E] [IsScalarTower F K E] {x : E} (hx : x Polynomial.aroots p E) [Fintype (K →ₐ[F] E)] [Fintype ({ x // x IntermediateField.restrictScalars F Kx } →ₐ[F] E)] :

                  Equivalent characterizations of a Galois extension of finite degree

                  instance IsGalois.normalClosure (k : Type u_1) (K : Type u_2) (F : Type u_3) [Field k] [Field K] [Field F] [Algebra k K] [Algebra k F] [Algebra K F] [IsScalarTower k K F] [IsGalois k F] :
                  IsGalois k { x // x normalClosure k K F }
                  Equations