Documentation

Mathlib.Algebra.Algebra.Tower

Towers of algebras #

In this file we prove basic facts about towers of algebra.

An algebra tower A/S/R is expressed by having instances of Algebra A S, Algebra R S, Algebra R A and IsScalarTower R S A, the later asserting the compatibility condition (r • s) • a = r • (s • a).

An important definition is toAlgHom R S A, the canonical R-algebra homomorphism S →ₐ[R] A.

def Algebra.lsmul (R : Type u) {A : Type w} (B : Type u₁) (M : Type v₁) [CommSemiring R] [Semiring A] [Semiring B] [Algebra R A] [Algebra R B] [AddCommMonoid M] [Module R M] [Module A M] [Module B M] [IsScalarTower R A M] [IsScalarTower R B M] [SMulCommClass A B M] :

The R-algebra morphism A → End (M) corresponding to the representation of the algebra A on the B-module M.

This is a stronger version of DistribMulAction.toLinearMap, and could also have been called Algebra.toModuleEnd.

The typeclasses correspond to the situation where the types act on each other as

R ----→ B
| ⟍     |
|   ⟍   |
↓     ↘ ↓
A ----→ M

where the diagram commutes, the action by R commutes with everything, and the action by A and B on M commute.

Typically this is most useful with B = R as Algebra.lsmul R R A : A →ₐ[R] Module.End R M. However this can be used to get the fact that left-multiplication by A is right A-linear, and vice versa, as

example : A →ₐ[R] Module.End Aᵐᵒᵖ A := Algebra.lsmul R Aᵐᵒᵖ A
example : Aᵐᵒᵖ →ₐ[R] Module.End A A := Algebra.lsmul R A A

respectively; though LinearMap.mulLeft and LinearMap.mulRight can also be used here.

Equations
  • One or more equations did not get rendered due to their size.
Instances For
    @[simp]
    theorem Algebra.lsmul_coe (R : Type u) {A : Type w} (B : Type u₁) (M : Type v₁) [CommSemiring R] [Semiring A] [Semiring B] [Algebra R A] [Algebra R B] [AddCommMonoid M] [Module R M] [Module A M] [Module B M] [IsScalarTower R A M] [IsScalarTower R B M] [SMulCommClass A B M] (a : A) :
    ((Algebra.lsmul R B M) a) = fun (x : M) => a x
    theorem IsScalarTower.algebraMap_smul {R : Type u} (A : Type w) {M : Type v₁} [CommSemiring R] [Semiring A] [Algebra R A] [MulAction A M] [SMul R M] [IsScalarTower R A M] (r : R) (x : M) :
    (algebraMap R A) r x = r x
    theorem IsScalarTower.of_algebraMap_smul {R : Type u} {A : Type w} {M : Type v₁} [CommSemiring R] [Semiring A] [Algebra R A] [MulAction A M] [SMul R M] (h : ∀ (r : R) (x : M), (algebraMap R A) r x = r x) :
    theorem IsScalarTower.of_compHom (R : Type u) (A : Type w) (M : Type v₁) [CommSemiring R] [Semiring A] [Algebra R A] [MulAction A M] :
    theorem IsScalarTower.of_algebraMap_eq {R : Type u} {S : Type v} {A : Type w} [CommSemiring R] [CommSemiring S] [Semiring A] [Algebra R S] [Algebra S A] [Algebra R A] (h : ∀ (x : R), (algebraMap R A) x = (algebraMap S A) ((algebraMap R S) x)) :
    theorem IsScalarTower.of_algebraMap_eq' {R : Type u} {S : Type v} {A : Type w} [CommSemiring R] [CommSemiring S] [Semiring A] [Algebra R S] [Algebra S A] [Algebra R A] (h : algebraMap R A = RingHom.comp (algebraMap S A) (algebraMap R S)) :

    See note [partially-applied ext lemmas].

    theorem IsScalarTower.algebraMap_apply (R : Type u) (S : Type v) (A : Type w) [CommSemiring R] [CommSemiring S] [Semiring A] [Algebra R S] [Algebra S A] [Algebra R A] [IsScalarTower R S A] (x : R) :
    (algebraMap R A) x = (algebraMap S A) ((algebraMap R S) x)
    theorem IsScalarTower.Algebra.ext {S : Type u} {A : Type v} [CommSemiring S] [Semiring A] (h1 : Algebra S A) (h2 : Algebra S A) (h : ∀ (r : S) (x : A), (let_fun I := h1; r x) = r x) :
    h1 = h2
    def IsScalarTower.toAlgHom (R : Type u) (S : Type v) (A : Type w) [CommSemiring R] [CommSemiring S] [Semiring A] [Algebra R S] [Algebra S A] [Algebra R A] [IsScalarTower R S A] :

    In a tower, the canonical map from the middle element to the top element is an algebra homomorphism over the bottom element.

    Equations
    Instances For
      theorem IsScalarTower.toAlgHom_apply (R : Type u) (S : Type v) (A : Type w) [CommSemiring R] [CommSemiring S] [Semiring A] [Algebra R S] [Algebra S A] [Algebra R A] [IsScalarTower R S A] (y : S) :
      @[simp]
      theorem IsScalarTower.coe_toAlgHom (R : Type u) (S : Type v) (A : Type w) [CommSemiring R] [CommSemiring S] [Semiring A] [Algebra R S] [Algebra S A] [Algebra R A] [IsScalarTower R S A] :
      @[simp]
      theorem IsScalarTower.coe_toAlgHom' (R : Type u) (S : Type v) (A : Type w) [CommSemiring R] [CommSemiring S] [Semiring A] [Algebra R S] [Algebra S A] [Algebra R A] [IsScalarTower R S A] :
      (IsScalarTower.toAlgHom R S A) = (algebraMap S A)
      @[simp]
      theorem AlgHom.map_algebraMap {R : Type u} {S : Type v} {A : Type w} {B : Type u₁} [CommSemiring R] [CommSemiring S] [Semiring A] [Semiring B] [Algebra R S] [Algebra S A] [Algebra S B] [Algebra R A] [Algebra R B] [IsScalarTower R S A] [IsScalarTower R S B] (f : A →ₐ[S] B) (r : R) :
      f ((algebraMap R A) r) = (algebraMap R B) r
      @[simp]
      theorem AlgHom.comp_algebraMap_of_tower (R : Type u) {S : Type v} {A : Type w} {B : Type u₁} [CommSemiring R] [CommSemiring S] [Semiring A] [Semiring B] [Algebra R S] [Algebra S A] [Algebra S B] [Algebra R A] [Algebra R B] [IsScalarTower R S A] [IsScalarTower R S B] (f : A →ₐ[S] B) :
      instance IsScalarTower.subsemiring {S : Type v} {A : Type w} [CommSemiring S] [Semiring A] [Algebra S A] (U : Subsemiring S) :
      IsScalarTower (U) S A
      Equations
      • =
      instance IsScalarTower.of_algHom {R : Type u_1} {A : Type u_2} {B : Type u_3} [CommSemiring R] [CommSemiring A] [CommSemiring B] [Algebra R A] [Algebra R B] (f : A →ₐ[R] B) :
      Equations
      • =
      def AlgHom.restrictScalars (R : Type u) {S : Type v} {A : Type w} {B : Type u₁} [CommSemiring R] [CommSemiring S] [Semiring A] [Semiring B] [Algebra R S] [Algebra S A] [Algebra S B] [Algebra R A] [Algebra R B] [IsScalarTower R S A] [IsScalarTower R S B] (f : A →ₐ[S] B) :

      R ⟶ S induces S-Alg ⥤ R-Alg

      Equations
      Instances For
        theorem AlgHom.restrictScalars_apply (R : Type u) {S : Type v} {A : Type w} {B : Type u₁} [CommSemiring R] [CommSemiring S] [Semiring A] [Semiring B] [Algebra R S] [Algebra S A] [Algebra S B] [Algebra R A] [Algebra R B] [IsScalarTower R S A] [IsScalarTower R S B] (f : A →ₐ[S] B) (x : A) :
        @[simp]
        theorem AlgHom.coe_restrictScalars (R : Type u) {S : Type v} {A : Type w} {B : Type u₁} [CommSemiring R] [CommSemiring S] [Semiring A] [Semiring B] [Algebra R S] [Algebra S A] [Algebra S B] [Algebra R A] [Algebra R B] [IsScalarTower R S A] [IsScalarTower R S B] (f : A →ₐ[S] B) :
        @[simp]
        theorem AlgHom.coe_restrictScalars' (R : Type u) {S : Type v} {A : Type w} {B : Type u₁} [CommSemiring R] [CommSemiring S] [Semiring A] [Semiring B] [Algebra R S] [Algebra S A] [Algebra S B] [Algebra R A] [Algebra R B] [IsScalarTower R S A] [IsScalarTower R S B] (f : A →ₐ[S] B) :
        def AlgEquiv.restrictScalars (R : Type u) {S : Type v} {A : Type w} {B : Type u₁} [CommSemiring R] [CommSemiring S] [Semiring A] [Semiring B] [Algebra R S] [Algebra S A] [Algebra S B] [Algebra R A] [Algebra R B] [IsScalarTower R S A] [IsScalarTower R S B] (f : A ≃ₐ[S] B) :

        R ⟶ S induces S-Alg ⥤ R-Alg

        Equations
        • AlgEquiv.restrictScalars R f = let __src := f; { toEquiv := __src.toEquiv, map_mul' := , map_add' := , commutes' := }
        Instances For
          theorem AlgEquiv.restrictScalars_apply (R : Type u) {S : Type v} {A : Type w} {B : Type u₁} [CommSemiring R] [CommSemiring S] [Semiring A] [Semiring B] [Algebra R S] [Algebra S A] [Algebra S B] [Algebra R A] [Algebra R B] [IsScalarTower R S A] [IsScalarTower R S B] (f : A ≃ₐ[S] B) (x : A) :
          @[simp]
          theorem AlgEquiv.coe_restrictScalars (R : Type u) {S : Type v} {A : Type w} {B : Type u₁} [CommSemiring R] [CommSemiring S] [Semiring A] [Semiring B] [Algebra R S] [Algebra S A] [Algebra S B] [Algebra R A] [Algebra R B] [IsScalarTower R S A] [IsScalarTower R S B] (f : A ≃ₐ[S] B) :
          @[simp]
          theorem AlgEquiv.coe_restrictScalars' (R : Type u) {S : Type v} {A : Type w} {B : Type u₁} [CommSemiring R] [CommSemiring S] [Semiring A] [Semiring B] [Algebra R S] [Algebra S A] [Algebra S B] [Algebra R A] [Algebra R B] [IsScalarTower R S A] [IsScalarTower R S B] (f : A ≃ₐ[S] B) :
          theorem Submodule.restrictScalars_span (R : Type u) (A : Type w) {M : Type v₁} [CommSemiring R] [Semiring A] [Algebra R A] [AddCommMonoid M] [Module R M] [Module A M] [IsScalarTower R A M] (hsur : Function.Surjective (algebraMap R A)) (X : Set M) :

          If A is an R-algebra such that the induced morphism R →+* A is surjective, then the R-module generated by a set X equals the A-module generated by X.

          theorem Submodule.coe_span_eq_span_of_surjective (R : Type u) (A : Type w) {M : Type v₁} [CommSemiring R] [Semiring A] [Algebra R A] [AddCommMonoid M] [Module R M] [Module A M] [IsScalarTower R A M] (h : Function.Surjective (algebraMap R A)) (s : Set M) :
          (Submodule.span A s) = (Submodule.span R s)
          theorem Submodule.smul_mem_span_smul_of_mem {R : Type u} {S : Type v} {A : Type w} [Semiring R] [Semiring S] [AddCommMonoid A] [Module R S] [Module S A] [Module R A] [IsScalarTower R S A] {s : Set S} {t : Set A} {k : S} (hks : k Submodule.span R s) {x : A} (hx : x t) :
          theorem Submodule.span_smul_of_span_eq_top {R : Type u} {S : Type v} {A : Type w} [Semiring R] [Semiring S] [AddCommMonoid A] [Module R S] [Module S A] [Module R A] [IsScalarTower R S A] {s : Set S} (hs : Submodule.span R s = ) (t : Set A) :
          theorem Submodule.smul_mem_span_smul' {R : Type u} {S : Type v} {A : Type w} [Semiring R] [Semiring S] [AddCommMonoid A] [Module R S] [Module S A] [Module R A] [IsScalarTower R S A] {s : Set S} (hs : Submodule.span R s = ) {t : Set A} {k : S} {x : A} (hx : x Submodule.span R (s t)) :
          theorem Submodule.smul_mem_span_smul {R : Type u} {S : Type v} {A : Type w} [Semiring R] [Semiring S] [AddCommMonoid A] [Module R S] [Module S A] [Module R A] [IsScalarTower R S A] {s : Set S} (hs : Submodule.span R s = ) {t : Set A} {k : S} {x : A} (hx : x Submodule.span R t) :
          theorem Submodule.span_algebraMap_image_of_tower {R : Type u} [CommSemiring R] {S : Type u_1} {T : Type u_2} [CommSemiring S] [Semiring T] [Module R S] [Algebra R T] [Algebra S T] [IsScalarTower R S T] (a : Set S) :
          theorem Submodule.map_mem_span_algebraMap_image {R : Type u} [CommSemiring R] {S : Type u_1} {T : Type u_2} [CommSemiring S] [Semiring T] [Algebra R S] [Algebra R T] [Algebra S T] [IsScalarTower R S T] (x : S) (a : Set S) (hx : x Submodule.span R a) :
          (algebraMap S T) x Submodule.span R ((algebraMap S T) '' a)
          theorem Algebra.lsmul_injective (R : Type u) (A : Type w) (B : Type u₁) (M : Type v₁) [CommSemiring R] [Semiring A] [Semiring B] [Algebra R A] [Algebra R B] [AddCommGroup M] [Module R M] [Module A M] [Module B M] [IsScalarTower R A M] [IsScalarTower R B M] [SMulCommClass A B M] [NoZeroSMulDivisors A M] {x : A} (hx : x 0) :