Induced monoidal structure on Action V G
#
We show:
- When
V
is monoidal, braided, or symmetric, so isAction V G
.
Equations
- Action.instMonoidalCategory = CategoryTheory.Monoidal.transport (Action.functorCategoryEquivalence V G).symm
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
Equations
Equations
- ⋯ = ⋯
Equations
- ⋯ = ⋯
Upgrading the functor Action V G ⥤ (SingleObj G ⥤ V)
to a monoidal functor.
Equations
- Action.instMonoidalFunctorSingleObjαMonoidFunctor V G = inferInstanceAs (CategoryTheory.Monoidal.equivalenceTransported (Action.functorCategoryEquivalence V G).symm).inverse.Monoidal
Equations
- Action.instMonoidalFunctorSingleObjαMonoidFunctorFunctorCategoryEquivalence V G = id inferInstance
Upgrading the functor (SingleObj G ⥤ V) ⥤ Action V G
to a monoidal functor.
Equations
- Action.instMonoidalFunctorSingleObjαMonoidInverse V G = inferInstanceAs (CategoryTheory.Monoidal.equivalenceTransported (Action.functorCategoryEquivalence V G).symm).functor.Monoidal
Equations
- Action.instMonoidalFunctorSingleObjαMonoidInverseFunctorCategoryEquivalence V G = id inferInstance
Equations
- Action.instRightRigidCategoryFunctorSingleObjαMonoidObjGrpMonCatForget₂ V H = inferInstance
If V
is right rigid, so is Action V G
.
Equations
- One or more equations did not get rendered due to their size.
Equations
- Action.instLeftRigidCategoryFunctorSingleObjαMonoidObjGrpMonCatForget₂ V H = inferInstance
If V
is left rigid, so is Action V G
.
Equations
- One or more equations did not get rendered due to their size.
Equations
- Action.instRigidCategoryFunctorSingleObjαMonoidObjGrpMonCatForget₂ V H = inferInstance
If V
is rigid, so is Action V G
.
Equations
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
The natural isomorphism of G
-sets Gⁿ⁺¹ ≅ G × Gⁿ
, where G
acts by left multiplication on
each factor.
Equations
- Action.diagonalSucc G n = Action.mkIso (Fin.consEquiv fun (a : Fin (n + 1)) => G).symm.toIso ⋯
Instances For
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.
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.
A monoidal functor induces a monoidal functor between
the categories of G
-actions within those categories.
Equations
- F.instMonoidalActionMapAction = CategoryTheory.Functor.Monoidal.mk ⋯ ⋯ ⋯ ⋯