Documentation

Mathlib.RingTheory.IntegralRestrict

Restriction of various maps between fields to integrally closed subrings. #

In this file, we assume A is an integrally closed domain; K is the fraction ring of A; L is a finite (separable) extension of K; B is the integral closure of A in L. We call this the AKLB setup.

Main definition #

noncomputable def galLift (A : Type u_1) (K : Type u_2) (L : Type u_3) (B : Type u_4) [CommRing A] [CommRing B] [Algebra A B] [Field K] [Field L] [Algebra A K] [IsFractionRing A K] [Algebra B L] [Algebra K L] [Algebra A L] [IsScalarTower A B L] [IsScalarTower A K L] [IsIntegralClosure B A L] [FiniteDimensional K L] (σ : B →ₐ[A] B) :

The lift End(B/A) → End(L/K) in an ALKB setup. This is inverse to the restriction. See galRestrictHom.

Equations
Instances For
    noncomputable def galRestrictHom (A : Type u_1) (K : Type u_2) (L : Type u_3) (B : Type u_4) [CommRing A] [CommRing B] [Algebra A B] [Field K] [Field L] [Algebra A K] [IsFractionRing A K] [Algebra B L] [Algebra K L] [Algebra A L] [IsScalarTower A B L] [IsScalarTower A K L] [IsIntegralClosure B A L] [FiniteDimensional K L] :
    (L →ₐ[K] L) ≃* (B →ₐ[A] B)

    The restriction End(L/K) → End(B/A) in an AKLB setup. Also see galRestrict for the AlgEquiv version.

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      @[simp]
      theorem algebraMap_galRestrictHom_apply (A : Type u_1) (K : Type u_2) (L : Type u_3) (B : Type u_4) [CommRing A] [CommRing B] [Algebra A B] [Field K] [Field L] [Algebra A K] [IsFractionRing A K] [Algebra B L] [Algebra K L] [Algebra A L] [IsScalarTower A B L] [IsScalarTower A K L] [IsIntegralClosure B A L] [FiniteDimensional K L] (σ : L →ₐ[K] L) (x : B) :
      (algebraMap B L) (((galRestrictHom A K L B) σ) x) = σ ((algebraMap B L) x)
      @[simp]
      theorem galRestrictHom_symm_algebraMap_apply (A : Type u_1) (K : Type u_2) (L : Type u_3) (B : Type u_4) [CommRing A] [CommRing B] [Algebra A B] [Field K] [Field L] [Algebra A K] [IsFractionRing A K] [Algebra B L] [Algebra K L] [Algebra A L] [IsScalarTower A B L] [IsScalarTower A K L] [IsIntegralClosure B A L] [FiniteDimensional K L] (σ : B →ₐ[A] B) (x : B) :
      ((galRestrictHom A K L B).symm σ) ((algebraMap B L) x) = (algebraMap B L) (σ x)
      noncomputable def galRestrict (A : Type u_1) (K : Type u_2) (L : Type u_3) (B : Type u_4) [CommRing A] [CommRing B] [Algebra A B] [Field K] [Field L] [Algebra A K] [IsFractionRing A K] [Algebra B L] [Algebra K L] [Algebra A L] [IsScalarTower A B L] [IsScalarTower A K L] [IsIntegralClosure B A L] [FiniteDimensional K L] :
      (L ≃ₐ[K] L) ≃* B ≃ₐ[A] B

      The restriction Aut(L/K) → Aut(B/A) in an AKLB setup.

      Equations
      Instances For
        theorem coe_galRestrict_apply (A : Type u_1) {K : Type u_2} {L : Type u_3} (B : Type u_4) [CommRing A] [CommRing B] [Algebra A B] [Field K] [Field L] [Algebra A K] [IsFractionRing A K] [Algebra B L] [Algebra K L] [Algebra A L] [IsScalarTower A B L] [IsScalarTower A K L] [IsIntegralClosure B A L] [FiniteDimensional K L] (σ : L ≃ₐ[K] L) :
        ((galRestrict A K L B) σ) = (galRestrictHom A K L B) σ
        theorem galRestrict_apply (A : Type u_1) {K : Type u_2} {L : Type u_3} {B : Type u_4} [CommRing A] [CommRing B] [Algebra A B] [Field K] [Field L] [Algebra A K] [IsFractionRing A K] [Algebra B L] [Algebra K L] [Algebra A L] [IsScalarTower A B L] [IsScalarTower A K L] [IsIntegralClosure B A L] [FiniteDimensional K L] (σ : L ≃ₐ[K] L) (x : B) :
        ((galRestrict A K L B) σ) x = ((galRestrictHom A K L B) σ) x
        theorem algebraMap_galRestrict_apply (A : Type u_1) {K : Type u_2} {L : Type u_3} {B : Type u_4} [CommRing A] [CommRing B] [Algebra A B] [Field K] [Field L] [Algebra A K] [IsFractionRing A K] [Algebra B L] [Algebra K L] [Algebra A L] [IsScalarTower A B L] [IsScalarTower A K L] [IsIntegralClosure B A L] [FiniteDimensional K L] (σ : L ≃ₐ[K] L) (x : B) :
        (algebraMap B L) (((galRestrict A K L B) σ) x) = σ ((algebraMap B L) x)
        theorem prod_galRestrict_eq_norm (A : Type u_1) (K : Type u_2) (L : Type u_3) (B : Type u_4) [CommRing A] [CommRing B] [Algebra A B] [Field K] [Field L] [Algebra A K] [IsFractionRing A K] [Algebra B L] [Algebra K L] [Algebra A L] [IsScalarTower A B L] [IsScalarTower A K L] [IsIntegralClosure B A L] [FiniteDimensional K L] [IsGalois K L] [IsIntegrallyClosed A] (x : B) :
        (Finset.univ.prod fun (σ : L ≃ₐ[K] L) => ((galRestrict A K L B) σ) x) = (algebraMap A B) (IsIntegralClosure.mk' A ((Algebra.norm K) ((algebraMap B L) x)) )
        Equations
        • One or more equations did not get rendered due to their size.
        noncomputable def Algebra.intTraceAux (A : Type u_1) (K : Type u_2) (L : Type u_3) (B : Type u_4) [CommRing A] [CommRing B] [Algebra A B] [Field K] [Field L] [Algebra A K] [IsFractionRing A K] [Algebra B L] [Algebra K L] [Algebra A L] [IsScalarTower A B L] [IsScalarTower A K L] [IsIntegralClosure B A L] [FiniteDimensional K L] [IsIntegrallyClosed A] :

        The restriction of the trace on L/K restricted onto B/A in an AKLB setup. See Algebra.intTrace instead.

        Equations
        • One or more equations did not get rendered due to their size.
        Instances For
          theorem Algebra.map_intTraceAux {A : Type u_1} {K : Type u_2} {L : Type u_3} {B : Type u_4} [CommRing A] [CommRing B] [Algebra A B] [Field K] [Field L] [Algebra A K] [IsFractionRing A K] [Algebra B L] [Algebra K L] [Algebra A L] [IsScalarTower A B L] [IsScalarTower A K L] [IsIntegralClosure B A L] [FiniteDimensional K L] [IsIntegrallyClosed A] (x : B) :
          (algebraMap A K) ((Algebra.intTraceAux A K L B) x) = (Algebra.trace K L) ((algebraMap B L) x)
          noncomputable def Algebra.intTrace (A : Type u_1) (B : Type u_4) [CommRing A] [CommRing B] [Algebra A B] [IsDomain A] [IsIntegrallyClosed A] [IsDomain B] [IsIntegrallyClosed B] [Module.Finite A B] [NoZeroSMulDivisors A B] :

          The trace of a finite extension of integrally closed domains B/A is the restriction of the trace on Frac(B)/Frac(A) onto B/A. See Algebra.algebraMap_intTrace.

          Equations
          Instances For
            theorem Algebra.algebraMap_intTrace {A : Type u_1} {K : Type u_2} {L : Type u_3} {B : Type u_4} [CommRing A] [CommRing B] [Algebra A B] [Field K] [Field L] [Algebra A K] [IsFractionRing A K] [Algebra B L] [Algebra K L] [Algebra A L] [IsScalarTower A B L] [IsScalarTower A K L] [IsIntegralClosure B A L] [FiniteDimensional K L] [IsDomain A] [IsIntegrallyClosed A] [IsDomain B] [IsIntegrallyClosed B] [Module.Finite A B] [NoZeroSMulDivisors A B] (x : B) :
            (algebraMap A K) ((Algebra.intTrace A B) x) = (Algebra.trace K L) ((algebraMap B L) x)
            theorem Algebra.intTrace_eq_of_isLocalization (A : Type u_1) (B : Type u_4) [CommRing A] [CommRing B] [Algebra A B] {Aₘ : Type u_5} {Bₘ : Type u_6} [CommRing Aₘ] [CommRing Bₘ] [Algebra Aₘ Bₘ] [Algebra A Aₘ] [Algebra B Bₘ] [Algebra A Bₘ] [IsScalarTower A Aₘ Bₘ] [IsScalarTower A B Bₘ] (M : Submonoid A) [IsLocalization M Aₘ] [IsLocalization (Algebra.algebraMapSubmonoid B M) Bₘ] [IsDomain A] [IsIntegrallyClosed A] [IsDomain B] [IsIntegrallyClosed B] [Module.Finite A B] [NoZeroSMulDivisors A B] [IsDomain Aₘ] [IsIntegrallyClosed Aₘ] [IsDomain Bₘ] [IsIntegrallyClosed Bₘ] [NoZeroSMulDivisors Aₘ Bₘ] [Module.Finite Aₘ Bₘ] (x : B) :
            (algebraMap A Aₘ) ((Algebra.intTrace A B) x) = (Algebra.intTrace Aₘ Bₘ) ((algebraMap B Bₘ) x)
            noncomputable def Algebra.intNormAux (A : Type u_1) (K : Type u_2) (L : Type u_3) (B : Type u_4) [CommRing A] [CommRing B] [Algebra A B] [Field K] [Field L] [Algebra A K] [IsFractionRing A K] [Algebra B L] [Algebra K L] [Algebra A L] [IsScalarTower A B L] [IsScalarTower A K L] [IsIntegralClosure B A L] [FiniteDimensional K L] [IsIntegrallyClosed A] [IsSeparable K L] :
            B →* A

            The restriction of the norm on L/K restricted onto B/A in an AKLB setup. See Algebra.intNorm instead.

            Equations
            Instances For
              theorem Algebra.map_intNormAux {A : Type u_1} {K : Type u_2} {L : Type u_3} {B : Type u_4} [CommRing A] [CommRing B] [Algebra A B] [Field K] [Field L] [Algebra A K] [IsFractionRing A K] [Algebra B L] [Algebra K L] [Algebra A L] [IsScalarTower A B L] [IsScalarTower A K L] [IsIntegralClosure B A L] [FiniteDimensional K L] [IsIntegrallyClosed A] [IsSeparable K L] (x : B) :
              (algebraMap A K) ((Algebra.intNormAux A K L B) x) = (Algebra.norm K) ((algebraMap B L) x)

              The norm of a finite extension of integrally closed domains B/A is the restriction of the norm on Frac(B)/Frac(A) onto B/A. See Algebra.algebraMap_intNorm.

              Equations
              Instances For
                theorem Algebra.algebraMap_intNorm {A : Type u_1} {K : Type u_2} {L : Type u_3} {B : Type u_4} [CommRing A] [CommRing B] [Algebra A B] [Field K] [Field L] [Algebra A K] [IsFractionRing A K] [Algebra B L] [Algebra K L] [Algebra A L] [IsScalarTower A B L] [IsScalarTower A K L] [IsIntegralClosure B A L] [FiniteDimensional K L] [IsDomain A] [IsIntegrallyClosed A] [IsDomain B] [IsIntegrallyClosed B] [Module.Finite A B] [NoZeroSMulDivisors A B] [IsSeparable (FractionRing A) (FractionRing B)] (x : B) :
                (algebraMap A K) ((Algebra.intNorm A B) x) = (Algebra.norm K) ((algebraMap B L) x)
                theorem Algebra.intNorm_eq_of_isLocalization {A : Type u_1} {B : Type u_4} [CommRing A] [CommRing B] [Algebra A B] {Aₘ : Type u_5} {Bₘ : Type u_6} [CommRing Aₘ] [CommRing Bₘ] [Algebra Aₘ Bₘ] [Algebra A Aₘ] [Algebra B Bₘ] [Algebra A Bₘ] [IsScalarTower A Aₘ Bₘ] [IsScalarTower A B Bₘ] (M : Submonoid A) [IsLocalization M Aₘ] [IsLocalization (Algebra.algebraMapSubmonoid B M) Bₘ] [IsDomain A] [IsIntegrallyClosed A] [IsDomain B] [IsIntegrallyClosed B] [Module.Finite A B] [NoZeroSMulDivisors A B] [IsSeparable (FractionRing A) (FractionRing B)] [IsDomain Aₘ] [IsIntegrallyClosed Aₘ] [IsDomain Bₘ] [IsIntegrallyClosed Bₘ] [NoZeroSMulDivisors Aₘ Bₘ] [Module.Finite Aₘ Bₘ] [IsSeparable (FractionRing Aₘ) (FractionRing Bₘ)] (x : B) :
                (algebraMap A Aₘ) ((Algebra.intNorm A B) x) = (Algebra.intNorm Aₘ Bₘ) ((algebraMap B Bₘ) x)
                theorem Algebra.algebraMap_intNorm_of_isGalois (A : Type u_1) (B : Type u_4) [CommRing A] [CommRing B] [Algebra A B] [IsDomain A] [IsIntegrallyClosed A] [IsDomain B] [IsIntegrallyClosed B] [Module.Finite A B] [NoZeroSMulDivisors A B] [IsGalois (FractionRing A) (FractionRing B)] {x : B} :
                (algebraMap A B) ((Algebra.intNorm A B) x) = Finset.univ.prod fun (σ : B ≃ₐ[A] B) => σ x