Documentation

Mathlib.CategoryTheory.Action.Limits

Categorical properties of Action V G #

We show:

F : C ⥤ Action V G preserves the limit of some K : J ⥤ C if if it does after postcomposing with the forgetful functor Action V G ⥤ V.

F : C ⥤ Action V G preserves limits of some shape J if it does after postcomposing with the forgetful functor Action V G ⥤ V.

F : C ⥤ Action V G preserves the colimit of some K : J ⥤ C if if it does after postcomposing with the forgetful functor Action V G ⥤ V.

F : C ⥤ Action V G preserves colimits of some shape J if it does after postcomposing with the forgetful functor Action V G ⥤ V.

Equations
instance Action.instAddHom {V : Type (u + 1)} [CategoryTheory.LargeCategory V] {G : MonCat} [CategoryTheory.Preadditive V] {X Y : Action V G} :
Add (X Y)
Equations
instance Action.instNegHom {V : Type (u + 1)} [CategoryTheory.LargeCategory V] {G : MonCat} [CategoryTheory.Preadditive V] {X Y : Action V G} :
Neg (X Y)
Equations
Equations
@[simp]
theorem Action.neg_hom {V : Type (u + 1)} [CategoryTheory.LargeCategory V] {G : MonCat} [CategoryTheory.Preadditive V] {X Y : Action V G} (f : X Y) :
(-f).hom = -f.hom
@[simp]
theorem Action.add_hom {V : Type (u + 1)} [CategoryTheory.LargeCategory V] {G : MonCat} [CategoryTheory.Preadditive V] {X Y : Action V G} (f g : X Y) :
(f + g).hom = f.hom + g.hom
@[simp]
theorem Action.sum_hom {V : Type (u + 1)} [CategoryTheory.LargeCategory V] {G : MonCat} [CategoryTheory.Preadditive V] {X Y : Action V G} {ι : Type u_1} (f : ι(X Y)) (s : Finset ι) :
(s.sum f).hom = is, (f i).hom
Equations
@[simp]
theorem Action.smul_hom {V : Type (u + 1)} [CategoryTheory.LargeCategory V] {G : MonCat} [CategoryTheory.Preadditive V] {R : Type u_1} [Semiring R] [CategoryTheory.Linear R V] {X Y : Action V G} (r : R) (f : X Y) :
(r f).hom = r f.hom
instance Action.res_additive {V : Type (u + 1)} [CategoryTheory.LargeCategory V] {G : MonCat} [CategoryTheory.Preadditive V] {H : MonCat} (f : G H) :
(res V f).Additive

Auxiliary construction for the Abelian (Action V G) instance.

Equations
Instances For
    instance CategoryTheory.Functor.mapAction_preadditive {V : Type (u + 1)} [LargeCategory V] {W : Type (u + 1)} [LargeCategory W] (F : Functor V W) (G : MonCat) [Preadditive V] [Preadditive W] [F.Additive] :
    (F.mapAction G).Additive
    instance CategoryTheory.Functor.mapAction_linear {V : Type (u + 1)} [LargeCategory V] {W : Type (u + 1)} [LargeCategory W] (F : Functor V W) (G : MonCat) [Preadditive V] [Preadditive W] {R : Type u_1} [Semiring R] [CategoryTheory.Linear R V] [CategoryTheory.Linear R W] [F.Additive] [Linear R F] :
    Linear R (F.mapAction G)