Documentation

Mathlib.CategoryTheory.Monoidal.Action.Basic

Left actions from a monoidal category on a category #

Given a monoidal category C, and a category D, we define a left action of C on D as the data of an object c ⊙ₗ d of D for every c : C and d : D, as well as the data required to turn - ⊙ₗ - into a bifunctor, along with structure natural isomorphisms (- ⊗ -) ⊙ₗ - ≅ - ⊙ₗ - ⊙ₗ - and 𝟙_ C ⊙ₗ - ≅ -, subject to coherence conditions.

References #

TODOs/Projects #

A class that carries the non-Prop data required to define a left action of a monoidal category C on a category D, to set up notations.

  • actionObj : CDD

    The left action on objects. This is denoted c ⊙ₗ d.

  • actionHomLeft {c c' : C} (f : c c') (d : D) : actionObj c d actionObj c' d

    The left action of a map f : c ⟶ c' in C on an object d in D. If we are to consider the action as a functor Α : C ⥤ D ⥤ D, this is (Α.map f).app d. This is denoted f ⊵ₗ d`

  • actionHomRight (c : C) {d d' : D} (f : d d') : actionObj c d actionObj c d'

    The action of an object c : C on a map f : d ⟶ d' in D. If we are to consider the action as a functor Α : C ⥤ D ⥤ D, this is (Α.obj c).map f. This is denoted c ⊴ₗ f`.

  • actionHom {c c' : C} {d d' : D} (f : c c') (g : d d') : actionObj c d actionObj c' d'

    The action of a pair of maps f : c ⟶ c' and d ⟶ d'. By default, this is defined in terms of actionHomLeft and actionHomRight.

  • actionAssocIso (c c' : C) (d : D) : actionObj (tensorObj c c') d actionObj c (actionObj c' d)

    The structural isomorphism (c ⊗ c') ⊙ₗ d ≅ c ⊙ₗ (c' ⊙ₗ d).

  • actionUnitIso (d : D) : actionObj (tensorUnit C) d d

    The structural isomorphism between 𝟙_ C ⊙ₗ d and d.

Instances

    Notation for actionObj, the action of C on D.

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

      Notation for actionHomLeft, the action of C on morphisms in D.

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

        Notation for actionHomRight, the action of morphism in C on D.

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

          Notation for actionHom, the bifunctorial action of morphisms in C and D on - ⊙ₗ -.

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

            Notation for actionAssocIso, the structural isomorphism - ⊗ - ⊙ₗ - ≅ - ⊙ₗ - ⊙ₗ -.

            Equations
            Instances For

              Notation for actionUnitIso, the structural isomorphism 𝟙_ C ⊙ₗ - ≅ -.

              Equations
              Instances For

                Notation for actionUnitIso, the structural isomorphism 𝟙_ C ⊙ₗ - ≅ -, allowing one to specify the acting category.

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

                  A MonoidalLeftAction C D is is the data of:

                  • For every object c : C and d : D, an object c ⊙ₗ d of D.
                  • For every morphism f : (c : C) ⟶ c' and every d : D, a morphism f ⊵ₗ d : c ⊙ₗ d ⟶ c' ⊙ₗ d.
                  • For every morphism f : (d : D) ⟶ d' and every c : C, a morphism c ⊴ₗ f : c ⊙ₗ d ⟶ c ⊙ₗ d'.
                  • For every pair of morphisms f : (c : C) ⟶ c' and f : (d : D) ⟶ d', a morphism f ⊙ₗ f' : c ⊙ₗ d ⟶ c' ⊙ₗ d'.
                  • A structure isomorphism αₗ c c' d : c ⊗ c' ⊙ₗ d ≅ c ⊙ₗ c' ⊙ₗ d.
                  • A structure isomorphism λₗ d : (𝟙_ C) ⊙ₗ d ≅ d. Furthermore, we require identities that turn - ⊙ₗ - into a bifunctor, ensure naturality of αₗ and λₗ, and ensure compatibilies with the associator and unitor isomorphisms in C.
                  Instances
                    theorem CategoryTheory.MonoidalCategory.MonoidalLeftAction.actionHom_def_assoc {C : Type u_1} {D : Type u_2} {inst✝ : Category.{u_3, u_1} C} {inst✝¹ : Category.{u_4, u_2} D} {inst✝² : MonoidalCategory C} [self : MonoidalLeftAction C D] {c c' : C} {d d' : D} (f : c c') (g : d d') {Z : D} (h : actionObj c' d' Z) :
                    theorem CategoryTheory.MonoidalCategory.MonoidalLeftAction.id_actionHomLeft_assoc {C : Type u_1} {D : Type u_2} {inst✝ : Category.{u_3, u_1} C} {inst✝¹ : Category.{u_4, u_2} D} {inst✝² : MonoidalCategory C} [self : MonoidalLeftAction C D] (c : C) (d : D) {Z : D} (h : actionObj c d Z) :
                    theorem CategoryTheory.MonoidalCategory.MonoidalLeftAction.actionHom_comp_assoc {C : Type u_1} {D : Type u_2} {inst✝ : Category.{u_3, u_1} C} {inst✝¹ : Category.{u_4, u_2} D} {inst✝² : MonoidalCategory C} [self : MonoidalLeftAction C D] {c c' c'' : C} {d d' d'' : D} (f₁ : c c') (f₂ : c' c'') (g₁ : d d') (g₂ : d' d'') {Z : D} (h : actionObj c'' d'' Z) :
                    theorem CategoryTheory.MonoidalCategory.MonoidalLeftAction.actionAssocIso_hom_naturality_assoc {C : Type u_1} {D : Type u_2} {inst✝ : Category.{u_3, u_1} C} {inst✝¹ : Category.{u_4, u_2} D} {inst✝² : MonoidalCategory C} [self : MonoidalLeftAction C D] {c₁ c₂ c₃ c₄ : C} {d₁ d₂ : D} (f : c₁ c₂) (g : c₃ c₄) (h : d₁ d₂) {Z : D} (h✝ : actionObj c₂ (actionObj c₄ d₂) Z) :
                    @[simp]
                    theorem CategoryTheory.MonoidalCategory.MonoidalLeftAction.associator_actionHom_assoc {C : Type u_1} {D : Type u_2} {inst✝ : Category.{u_3, u_1} C} {inst✝¹ : Category.{u_4, u_2} D} {inst✝² : MonoidalCategory C} [self : MonoidalLeftAction C D] (c₁ c₂ c₃ : C) (d : D) {Z : D} (h : actionObj c₁ (actionObj c₂ (actionObj c₃ d)) Z) :

                    A monoidal category acts on itself through the tensor product.

                    Equations
                    • One or more equations did not get rendered due to their size.
                    @[simp]
                    theorem CategoryTheory.MonoidalCategory.selfAction_actionHom (C : Type u_1) [Category.{u_3, u_1} C] [MonoidalCategory C] {c✝ c'✝ d✝ d'✝ : C} (f : c✝ c'✝) (g : d✝ d'✝) :
                    theorem CategoryTheory.MonoidalCategory.MonoidalLeftAction.actionHom_def' {C : Type u_1} {D : Type u_2} [Category.{u_3, u_1} C] [Category.{u_4, u_2} D] [MonoidalCategory C] [MonoidalLeftAction C D] {x₁ y₁ : C} {x₂ y₂ : D} (f : x₁ y₁) (g : x₂ y₂) :
                    theorem CategoryTheory.MonoidalCategory.MonoidalLeftAction.actionHom_def'_assoc {C : Type u_1} {D : Type u_2} [Category.{u_3, u_1} C] [Category.{u_4, u_2} D] [MonoidalCategory C] [MonoidalLeftAction C D] {x₁ y₁ : C} {x₂ y₂ : D} (f : x₁ y₁) (g : x₂ y₂) {Z : D} (h : actionObj y₁ y₂ Z) :
                    theorem CategoryTheory.MonoidalCategory.MonoidalLeftAction.actionAssocIso_inv_naturality {C : Type u_1} {D : Type u_2} [Category.{u_3, u_1} C] [Category.{u_4, u_2} D] [MonoidalCategory C] [MonoidalLeftAction C D] {c₁ c₂ c₃ c₄ : C} {d₁ d₂ : D} (f : c₁ c₂) (g : c₃ c₄) (h : d₁ d₂) :
                    theorem CategoryTheory.MonoidalCategory.MonoidalLeftAction.actionAssocIso_inv_naturality_assoc {C : Type u_1} {D : Type u_2} [Category.{u_3, u_1} C] [Category.{u_4, u_2} D] [MonoidalCategory C] [MonoidalLeftAction C D] {c₁ c₂ c₃ c₄ : C} {d₁ d₂ : D} (f : c₁ c₂) (g : c₃ c₄) (h : d₁ d₂) {Z : D} (h✝ : actionObj (tensorObj c₂ c₄) d₂ Z) :
                    @[simp]
                    theorem CategoryTheory.MonoidalCategory.MonoidalLeftAction.inv_actionHom {C : Type u_1} {D : Type u_2} [Category.{u_3, u_1} C] [Category.{u_4, u_2} D] [MonoidalCategory C] [MonoidalLeftAction C D] {x y : C} {x' y' : D} (f : x y) (g : x' y') [IsIso f] [IsIso g] :
                    inv (actionHom f g) = actionHom (inv f) (inv g)

                    Bundle the action of C on D as a functor C ⥤ D ⥤ D.

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

                      Bundle αₗ _ _ _ as an isomorphism of trifunctors.

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

                        Bundle λₗ _ as an isomorphism of functors.

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