Preadditive structure on algebras over a monad #
If C
is a preadditive category and F
is an additive endofunctor on C
then Algebra F
is
also preadditive. Dually, the category Coalgebra F
is also preadditive.
instance
CategoryTheory.Endofunctor.algebraPreadditive
(C : Type u₁)
[CategoryTheory.Category.{v₁, u₁} C]
[CategoryTheory.Preadditive C]
(F : CategoryTheory.Functor C C)
[F.Additive]
:
The category of algebras over an additive endofunctor on a preadditive category is preadditive.
Equations
- CategoryTheory.Endofunctor.algebraPreadditive C F = { homGroup := fun (A₁ A₂ : CategoryTheory.Endofunctor.Algebra F) => AddCommGroup.mk ⋯, add_comp := ⋯, comp_add := ⋯ }
@[simp]
theorem
CategoryTheory.Endofunctor.algebraPreadditive_homGroup_add_f
(C : Type u₁)
[CategoryTheory.Category.{v₁, u₁} C]
[CategoryTheory.Preadditive C]
(F : CategoryTheory.Functor C C)
[F.Additive]
(A₁ A₂ : CategoryTheory.Endofunctor.Algebra F)
(α β : A₁ ⟶ A₂)
:
@[simp]
theorem
CategoryTheory.Endofunctor.algebraPreadditive_homGroup_zero_f
(C : Type u₁)
[CategoryTheory.Category.{v₁, u₁} C]
[CategoryTheory.Preadditive C]
(F : CategoryTheory.Functor C C)
[F.Additive]
(A₁ A₂ : CategoryTheory.Endofunctor.Algebra F)
:
@[simp]
theorem
CategoryTheory.Endofunctor.algebraPreadditive_homGroup_neg_f
(C : Type u₁)
[CategoryTheory.Category.{v₁, u₁} C]
[CategoryTheory.Preadditive C]
(F : CategoryTheory.Functor C C)
[F.Additive]
(A₁ A₂ : CategoryTheory.Endofunctor.Algebra F)
(α : A₁ ⟶ A₂)
:
@[simp]
theorem
CategoryTheory.Endofunctor.algebraPreadditive_homGroup_zsmul_f
(C : Type u₁)
[CategoryTheory.Category.{v₁, u₁} C]
[CategoryTheory.Preadditive C]
(F : CategoryTheory.Functor C C)
[F.Additive]
(A₁ A₂ : CategoryTheory.Endofunctor.Algebra F)
(r : ℤ)
(α : A₁ ⟶ A₂)
:
@[simp]
theorem
CategoryTheory.Endofunctor.algebraPreadditive_homGroup_sub_f
(C : Type u₁)
[CategoryTheory.Category.{v₁, u₁} C]
[CategoryTheory.Preadditive C]
(F : CategoryTheory.Functor C C)
[F.Additive]
(A₁ A₂ : CategoryTheory.Endofunctor.Algebra F)
(α β : A₁ ⟶ A₂)
:
@[simp]
theorem
CategoryTheory.Endofunctor.algebraPreadditive_homGroup_nsmul_f
(C : Type u₁)
[CategoryTheory.Category.{v₁, u₁} C]
[CategoryTheory.Preadditive C]
(F : CategoryTheory.Functor C C)
[F.Additive]
(A₁ A₂ : CategoryTheory.Endofunctor.Algebra F)
(n : ℕ)
(α : A₁ ⟶ A₂)
:
instance
CategoryTheory.Algebra.forget_additive
(C : Type u₁)
[CategoryTheory.Category.{v₁, u₁} C]
[CategoryTheory.Preadditive C]
(F : CategoryTheory.Functor C C)
[F.Additive]
:
(CategoryTheory.Endofunctor.Algebra.forget F).Additive
Equations
- ⋯ = ⋯
instance
CategoryTheory.Endofunctor.coalgebraPreadditive
(C : Type u₁)
[CategoryTheory.Category.{v₁, u₁} C]
[CategoryTheory.Preadditive C]
(F : CategoryTheory.Functor C C)
[F.Additive]
:
Equations
- CategoryTheory.Endofunctor.coalgebraPreadditive C F = { homGroup := fun (A₁ A₂ : CategoryTheory.Endofunctor.Coalgebra F) => AddCommGroup.mk ⋯, add_comp := ⋯, comp_add := ⋯ }
@[simp]
theorem
CategoryTheory.Endofunctor.coalgebraPreadditive_homGroup_sub_f
(C : Type u₁)
[CategoryTheory.Category.{v₁, u₁} C]
[CategoryTheory.Preadditive C]
(F : CategoryTheory.Functor C C)
[F.Additive]
(A₁ A₂ : CategoryTheory.Endofunctor.Coalgebra F)
(α β : A₁ ⟶ A₂)
:
@[simp]
theorem
CategoryTheory.Endofunctor.coalgebraPreadditive_homGroup_add_f
(C : Type u₁)
[CategoryTheory.Category.{v₁, u₁} C]
[CategoryTheory.Preadditive C]
(F : CategoryTheory.Functor C C)
[F.Additive]
(A₁ A₂ : CategoryTheory.Endofunctor.Coalgebra F)
(α β : A₁ ⟶ A₂)
:
@[simp]
theorem
CategoryTheory.Endofunctor.coalgebraPreadditive_homGroup_neg_f
(C : Type u₁)
[CategoryTheory.Category.{v₁, u₁} C]
[CategoryTheory.Preadditive C]
(F : CategoryTheory.Functor C C)
[F.Additive]
(A₁ A₂ : CategoryTheory.Endofunctor.Coalgebra F)
(α : A₁ ⟶ A₂)
:
@[simp]
theorem
CategoryTheory.Endofunctor.coalgebraPreadditive_homGroup_zsmul_f
(C : Type u₁)
[CategoryTheory.Category.{v₁, u₁} C]
[CategoryTheory.Preadditive C]
(F : CategoryTheory.Functor C C)
[F.Additive]
(A₁ A₂ : CategoryTheory.Endofunctor.Coalgebra F)
(r : ℤ)
(α : A₁ ⟶ A₂)
:
@[simp]
theorem
CategoryTheory.Endofunctor.coalgebraPreadditive_homGroup_zero_f
(C : Type u₁)
[CategoryTheory.Category.{v₁, u₁} C]
[CategoryTheory.Preadditive C]
(F : CategoryTheory.Functor C C)
[F.Additive]
(A₁ A₂ : CategoryTheory.Endofunctor.Coalgebra F)
:
@[simp]
theorem
CategoryTheory.Endofunctor.coalgebraPreadditive_homGroup_nsmul_f
(C : Type u₁)
[CategoryTheory.Category.{v₁, u₁} C]
[CategoryTheory.Preadditive C]
(F : CategoryTheory.Functor C C)
[F.Additive]
(A₁ A₂ : CategoryTheory.Endofunctor.Coalgebra F)
(n : ℕ)
(α : A₁ ⟶ A₂)
:
instance
CategoryTheory.Coalgebra.forget_additive
(C : Type u₁)
[CategoryTheory.Category.{v₁, u₁} C]
[CategoryTheory.Preadditive C]
(F : CategoryTheory.Functor C C)
[F.Additive]
:
(CategoryTheory.Endofunctor.Coalgebra.forget F).Additive
Equations
- ⋯ = ⋯