Documentation

Mathlib.CategoryTheory.Action.Monoidal

Induced monoidal structure on Action V G #

We show:

@[simp]
theorem Action.instMonoidalCategory_tensorHom_hom {V : Type (u + 1)} [CategoryTheory.LargeCategory V] {G : MonCat} [CategoryTheory.MonoidalCategory V] {X₁✝ Y₁✝ X₂✝ Y₂✝ : Action V G} (f : X₁✝ Y₁✝) (g : X₂✝ Y₂✝) :
@[simp]
@[simp]
def Action.tensorUnitIso {V : Type (u + 1)} [CategoryTheory.LargeCategory V] {G : MonCat} [CategoryTheory.MonoidalCategory V] {X : V} (f : 𝟙_ V X) :
𝟙_ (Action V G) { V := X, ρ := 1 }

Given an object X isomorphic to the tensor unit of V, X equipped with the trivial action is isomorphic to the tensor unit of Action V G.

Equations
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.

    When V is braided the forgetful functor Action V G to V is braided.

    Equations

    If V is right rigid, so is Action V G.

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

    If V is left rigid, so is Action V G.

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

    Given X : Action (Type u) (MonCat.of G) for G a group, then G × X (with G acting as left multiplication on the first factor and by X.ρ on the second) is isomorphic as a G-set to G × X (with G acting as left multiplication on the first factor and trivially on the second). The isomorphism is given by (g, x) ↦ (g, g⁻¹ • x).

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      @[simp]
      theorem Action.leftRegularTensorIso_inv_hom (G : Type u) [Group G] (X : Action (Type u) (MonCat.of G)) (g : (CategoryTheory.MonoidalCategoryStruct.tensorObj (leftRegular G) { V := X.V, ρ := 1 }).V) :
      (leftRegularTensorIso G X).inv.hom g = (g.1, X g.1 g.2)
      @[simp]

      The natural isomorphism of G-sets Gⁿ⁺¹ ≅ G × Gⁿ, where G acts by left multiplication on each factor.

      Equations
      Instances For
        @[simp]
        theorem Action.diagonalSucc_inv_hom (G : Type u) [Monoid G] (n : ) (a✝ : (CategoryTheory.MonoidalCategoryStruct.tensorObj (leftRegular G) (diagonal G n)).V) :
        (diagonalSucc G n).inv.hom a✝ = (Fin.consEquiv fun (a : Fin (n + 1)) => G) a✝
        @[simp]
        theorem Action.diagonalSucc_hom_hom (G : Type u) [Monoid G] (n : ) (a✝ : (diagonal G (n + 1)).V) :
        (diagonalSucc G n).hom.hom a✝ = (Fin.consEquiv fun (a : Fin (n + 1)) => G).symm a✝
        instance CategoryTheory.Functor.instLaxMonoidalActionMapAction {V : Type (u + 1)} [LargeCategory V] {G : MonCat} {W : Type (u + 1)} [LargeCategory W] [MonoidalCategory V] [MonoidalCategory W] (F : Functor V W) [F.LaxMonoidal] :
        (F.mapAction G).LaxMonoidal

        A lax monoidal functor induces a lax monoidal functor between the categories of G-actions within those categories.

        Equations
        • One or more equations did not get rendered due to their size.
        @[simp]
        theorem CategoryTheory.Functor.mapAction_ε_hom {V : Type (u + 1)} [LargeCategory V] {G : MonCat} {W : Type (u + 1)} [LargeCategory W] [MonoidalCategory V] [MonoidalCategory W] (F : Functor V W) [F.LaxMonoidal] :
        (LaxMonoidal.ε (F.mapAction G)).hom = LaxMonoidal.ε F
        @[simp]
        theorem CategoryTheory.Functor.mapAction_μ_hom {V : Type (u + 1)} [LargeCategory V] {G : MonCat} {W : Type (u + 1)} [LargeCategory W] [MonoidalCategory V] [MonoidalCategory W] (F : Functor V W) [F.LaxMonoidal] (X Y : Action V G) :
        (LaxMonoidal.μ (F.mapAction G) X Y).hom = LaxMonoidal.μ F X.V Y.V
        instance CategoryTheory.Functor.instOplaxMonoidalActionMapAction {V : Type (u + 1)} [LargeCategory V] {G : MonCat} {W : Type (u + 1)} [LargeCategory W] [MonoidalCategory V] [MonoidalCategory W] (F : Functor V W) [F.OplaxMonoidal] :
        (F.mapAction G).OplaxMonoidal

        An oplax monoidal functor induces an oplax monoidal functor between the categories of G-actions within those categories.

        Equations
        • One or more equations did not get rendered due to their size.
        @[simp]
        theorem CategoryTheory.Functor.mapAction_η_hom {V : Type (u + 1)} [LargeCategory V] {G : MonCat} {W : Type (u + 1)} [LargeCategory W] [MonoidalCategory V] [MonoidalCategory W] (F : Functor V W) [F.OplaxMonoidal] :
        (OplaxMonoidal.η (F.mapAction G)).hom = OplaxMonoidal.η F
        @[simp]
        theorem CategoryTheory.Functor.mapAction_δ_hom {V : Type (u + 1)} [LargeCategory V] {G : MonCat} {W : Type (u + 1)} [LargeCategory W] [MonoidalCategory V] [MonoidalCategory W] (F : Functor V W) [F.OplaxMonoidal] (X Y : Action V G) :
        (OplaxMonoidal.δ (F.mapAction G) X Y).hom = OplaxMonoidal.δ F X.V Y.V
        instance CategoryTheory.Functor.instMonoidalActionMapAction {V : Type (u + 1)} [LargeCategory V] {G : MonCat} {W : Type (u + 1)} [LargeCategory W] [MonoidalCategory V] [MonoidalCategory W] (F : Functor V W) [F.Monoidal] :
        (F.mapAction G).Monoidal

        A monoidal functor induces a monoidal functor between the categories of G-actions within those categories.

        Equations