Documentation

Mathlib.CategoryTheory.Preadditive.EilenbergMoore

Preadditive structure on algebras over a monad #

If C is a preadditive category and T is an additive monad on C then Algebra T is also preadditive. Dually, if U is an additive comonad on C then Coalgebra U is preadditive as well.

@[simp]
theorem CategoryTheory.Monad.algebraPreadditive_homGroup_zsmul_f (C : Type u₁) [CategoryTheory.Category.{v₁, u₁} C] [CategoryTheory.Preadditive C] (T : CategoryTheory.Monad C) [T.Additive] (F : T.Algebra) (G : T.Algebra) (r : ) (α : F G) :
(r α).f = r α.f
@[simp]
theorem CategoryTheory.Monad.algebraPreadditive_homGroup_sub_f (C : Type u₁) [CategoryTheory.Category.{v₁, u₁} C] [CategoryTheory.Preadditive C] (T : CategoryTheory.Monad C) [T.Additive] (F : T.Algebra) (G : T.Algebra) (α : F G) (β : F G) :
(α - β).f = α.f - β.f
@[simp]
theorem CategoryTheory.Monad.algebraPreadditive_homGroup_neg_f (C : Type u₁) [CategoryTheory.Category.{v₁, u₁} C] [CategoryTheory.Preadditive C] (T : CategoryTheory.Monad C) [T.Additive] (F : T.Algebra) (G : T.Algebra) (α : F G) :
(-α).f = -α.f
@[simp]
theorem CategoryTheory.Monad.algebraPreadditive_homGroup_add_f (C : Type u₁) [CategoryTheory.Category.{v₁, u₁} C] [CategoryTheory.Preadditive C] (T : CategoryTheory.Monad C) [T.Additive] (F : T.Algebra) (G : T.Algebra) (α : F G) (β : F G) :
(α + β).f = α.f + β.f
@[simp]
theorem CategoryTheory.Monad.algebraPreadditive_homGroup_nsmul_f (C : Type u₁) [CategoryTheory.Category.{v₁, u₁} C] [CategoryTheory.Preadditive C] (T : CategoryTheory.Monad C) [T.Additive] (F : T.Algebra) (G : T.Algebra) (n : ) (α : F G) :
(n α).f = n α.f

The category of algebras over an additive monad on a preadditive category is preadditive.

Equations
Equations
  • =
@[simp]
theorem CategoryTheory.Comonad.coalgebraPreadditive_homGroup_neg_f (C : Type u₁) [CategoryTheory.Category.{v₁, u₁} C] [CategoryTheory.Preadditive C] (U : CategoryTheory.Comonad C) [U.Additive] (F : U.Coalgebra) (G : U.Coalgebra) (α : F G) :
(-α).f = -α.f
@[simp]
theorem CategoryTheory.Comonad.coalgebraPreadditive_homGroup_zsmul_f (C : Type u₁) [CategoryTheory.Category.{v₁, u₁} C] [CategoryTheory.Preadditive C] (U : CategoryTheory.Comonad C) [U.Additive] (F : U.Coalgebra) (G : U.Coalgebra) (r : ) (α : F G) :
(r α).f = r α.f
@[simp]
theorem CategoryTheory.Comonad.coalgebraPreadditive_homGroup_sub_f (C : Type u₁) [CategoryTheory.Category.{v₁, u₁} C] [CategoryTheory.Preadditive C] (U : CategoryTheory.Comonad C) [U.Additive] (F : U.Coalgebra) (G : U.Coalgebra) (α : F G) (β : F G) :
(α - β).f = α.f - β.f
@[simp]
theorem CategoryTheory.Comonad.coalgebraPreadditive_homGroup_nsmul_f (C : Type u₁) [CategoryTheory.Category.{v₁, u₁} C] [CategoryTheory.Preadditive C] (U : CategoryTheory.Comonad C) [U.Additive] (F : U.Coalgebra) (G : U.Coalgebra) (n : ) (α : F G) :
(n α).f = n α.f
@[simp]
theorem CategoryTheory.Comonad.coalgebraPreadditive_homGroup_add_f (C : Type u₁) [CategoryTheory.Category.{v₁, u₁} C] [CategoryTheory.Preadditive C] (U : CategoryTheory.Comonad C) [U.Additive] (F : U.Coalgebra) (G : U.Coalgebra) (α : F G) (β : F G) :
(α + β).f = α.f + β.f

The category of coalgebras over an additive comonad on a preadditive category is preadditive.

Equations
Equations
  • =