Documentation

Mathlib.Algebra.DirectSum.Algebra

Additively-graded algebra structures on ⨁ i, A i #

This file provides R-algebra structures on external direct sums of R-modules.

Recall that if A i are a family of AddCommMonoids indexed by an AddMonoid, then an instance of DirectSum.GMonoid A is a multiplication A i → A j → A (i + j) giving ⨁ i, A i the structure of a semiring. In this file, we introduce the DirectSum.GAlgebra R A class for the case where all A i are R-modules. This is the extra structure needed to promote ⨁ i, A i to an R-algebra.

Main definitions #

class DirectSum.GAlgebra {ι : Type uι} (R : Type uR) (A : ιType uA) [DecidableEq ι] [CommSemiring R] [(i : ι) → AddCommMonoid (A i)] [(i : ι) → Module R (A i)] [AddMonoid ι] [DirectSum.GSemiring A] :
Type (max uA uR)

A graded version of Algebra. An instance of DirectSum.GAlgebra R A endows (⨁ i, A i) with an R-algebra structure.

Instances
    instance GradedMonoid.smulCommClass_right {ι : Type uι} (R : Type uR) (A : ιType uA) [DecidableEq ι] [CommSemiring R] [(i : ι) → AddCommMonoid (A i)] [(i : ι) → Module R (A i)] [AddMonoid ι] [DirectSum.GSemiring A] [DirectSum.GAlgebra R A] :
    Equations
    • =
    instance GradedMonoid.isScalarTower_right {ι : Type uι} (R : Type uR) (A : ιType uA) [DecidableEq ι] [CommSemiring R] [(i : ι) → AddCommMonoid (A i)] [(i : ι) → Module R (A i)] [AddMonoid ι] [DirectSum.GSemiring A] [DirectSum.GAlgebra R A] :
    Equations
    • =
    instance DirectSum.instAlgebraDirectSumSemiring {ι : Type uι} (R : Type uR) (A : ιType uA) [DecidableEq ι] [CommSemiring R] [(i : ι) → AddCommMonoid (A i)] [(i : ι) → Module R (A i)] [AddMonoid ι] [DirectSum.GSemiring A] [DirectSum.GAlgebra R A] :
    Algebra R (DirectSum ι fun (i : ι) => A i)
    Equations
    • One or more equations did not get rendered due to their size.
    theorem DirectSum.algebraMap_apply {ι : Type uι} (R : Type uR) (A : ιType uA) [DecidableEq ι] [CommSemiring R] [(i : ι) → AddCommMonoid (A i)] [(i : ι) → Module R (A i)] [AddMonoid ι] [DirectSum.GSemiring A] [DirectSum.GAlgebra R A] (r : R) :
    (algebraMap R (DirectSum ι fun (i : ι) => A i)) r = (DirectSum.of A 0) (DirectSum.GAlgebra.toFun r)
    theorem DirectSum.algebraMap_toAddMonoid_hom {ι : Type uι} (R : Type uR) (A : ιType uA) [DecidableEq ι] [CommSemiring R] [(i : ι) → AddCommMonoid (A i)] [(i : ι) → Module R (A i)] [AddMonoid ι] [DirectSum.GSemiring A] [DirectSum.GAlgebra R A] :
    (algebraMap R (DirectSum ι fun (i : ι) => A i)) = AddMonoidHom.comp (DirectSum.of A 0) DirectSum.GAlgebra.toFun
    @[simp]
    theorem DirectSum.toAlgebra_apply {ι : Type uι} (R : Type uR) (A : ιType uA) {B : Type uB} [DecidableEq ι] [CommSemiring R] [(i : ι) → AddCommMonoid (A i)] [(i : ι) → Module R (A i)] [AddMonoid ι] [DirectSum.GSemiring A] [Semiring B] [DirectSum.GAlgebra R A] [Algebra R B] (f : (i : ι) → A i →ₗ[R] B) (hone : (f 0) GradedMonoid.GOne.one = 1) (hmul : ∀ {i j : ι} (ai : A i) (aj : A j), (f (i + j)) (GradedMonoid.GMul.mul ai aj) = (f i) ai * (f j) aj) (a : DirectSum ι fun (i : ι) => A i) :
    (DirectSum.toAlgebra R A f hone hmul) a = (DirectSum.toSemiring (fun (i : ι) => LinearMap.toAddMonoidHom (f i)) hone hmul) a
    def DirectSum.toAlgebra {ι : Type uι} (R : Type uR) (A : ιType uA) {B : Type uB} [DecidableEq ι] [CommSemiring R] [(i : ι) → AddCommMonoid (A i)] [(i : ι) → Module R (A i)] [AddMonoid ι] [DirectSum.GSemiring A] [Semiring B] [DirectSum.GAlgebra R A] [Algebra R B] (f : (i : ι) → A i →ₗ[R] B) (hone : (f 0) GradedMonoid.GOne.one = 1) (hmul : ∀ {i j : ι} (ai : A i) (aj : A j), (f (i + j)) (GradedMonoid.GMul.mul ai aj) = (f i) ai * (f j) aj) :
    (DirectSum ι fun (i : ι) => A i) →ₐ[R] B

    A family of LinearMaps preserving DirectSum.GOne.one and DirectSum.GMul.mul describes an AlgHom on ⨁ i, A i. This is a stronger version of DirectSum.toSemiring.

    Of particular interest is the case when A i are bundled subojects, f is the family of coercions such as Submodule.subtype (A i), and the [GMonoid A] structure originates from DirectSum.GMonoid.ofAddSubmodules, in which case the proofs about GOne and GMul can be discharged by rfl.

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      theorem DirectSum.algHom_ext' {ι : Type uι} (R : Type uR) (A : ιType uA) {B : Type uB} [DecidableEq ι] [CommSemiring R] [(i : ι) → AddCommMonoid (A i)] [(i : ι) → Module R (A i)] [AddMonoid ι] [DirectSum.GSemiring A] [Semiring B] [DirectSum.GAlgebra R A] [Algebra R B] ⦃f : (DirectSum ι fun (i : ι) => A i) →ₐ[R] B ⦃g : (DirectSum ι fun (i : ι) => A i) →ₐ[R] B (h : ∀ (i : ι), AlgHom.toLinearMap f ∘ₗ DirectSum.lof R ι A i = AlgHom.toLinearMap g ∘ₗ DirectSum.lof R ι A i) :
      f = g

      Two AlgHoms out of a direct sum are equal if they agree on the generators.

      See note [partially-applied ext lemmas].

      theorem DirectSum.algHom_ext {ι : Type uι} (R : Type uR) (A : ιType uA) {B : Type uB} [DecidableEq ι] [CommSemiring R] [(i : ι) → AddCommMonoid (A i)] [(i : ι) → Module R (A i)] [AddMonoid ι] [DirectSum.GSemiring A] [Semiring B] [DirectSum.GAlgebra R A] [Algebra R B] ⦃f : (DirectSum ι fun (i : ι) => A i) →ₐ[R] B ⦃g : (DirectSum ι fun (i : ι) => A i) →ₐ[R] B (h : ∀ (i : ι) (x : A i), f ((DirectSum.of A i) x) = g ((DirectSum.of A i) x)) :
      f = g
      @[simp]
      theorem DirectSum.gMulLHom_apply_apply {ι : Type uι} (R : Type uR) (A : ιType uA) [DecidableEq ι] [CommSemiring R] [(i : ι) → AddCommMonoid (A i)] [(i : ι) → Module R (A i)] [AddMonoid ι] [DirectSum.GSemiring A] [DirectSum.GAlgebra R A] {i : ι} {j : ι} (a : A i) (b : A j) :
      def DirectSum.gMulLHom {ι : Type uι} (R : Type uR) (A : ιType uA) [DecidableEq ι] [CommSemiring R] [(i : ι) → AddCommMonoid (A i)] [(i : ι) → Module R (A i)] [AddMonoid ι] [DirectSum.GSemiring A] [DirectSum.GAlgebra R A] {i : ι} {j : ι} :
      A i →ₗ[R] A j →ₗ[R] A (i + j)

      The piecewise multiplication from the Mul instance, as a bundled linear homomorphism.

      This is the graded version of LinearMap.mul, and the linear version of DirectSum.gMulHom

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

        Concrete instances #

        @[simp]
        theorem Algebra.directSumGAlgebra_toFun_apply {ι : Type uι} {R : Type u_1} {A : Type u_2} [DecidableEq ι] [AddMonoid ι] [CommSemiring R] [Semiring A] [Algebra R A] :
        ∀ (a : R), DirectSum.GAlgebra.toFun a = (algebraMap R A).toFun a
        instance Algebra.directSumGAlgebra {ι : Type uι} {R : Type u_1} {A : Type u_2} [DecidableEq ι] [AddMonoid ι] [CommSemiring R] [Semiring A] [Algebra R A] :
        DirectSum.GAlgebra R fun (x : ι) => A

        A direct sum of copies of an Algebra inherits the algebra structure.

        Equations