Additive Functors #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
A functor between two preadditive categories is called additive provided that the induced map on hom types is a morphism of abelian groups.
An additive functor between preadditive categories creates and preserves biproducts.
Conversely, if F : C ⥤ D
is a functor between preadditive categories, where C
has binary
biproducts, and if F
preserves binary biproducts, then F
is additive.
We also define the category of bundled additive functors.
Implementation details #
functor.additive
is a Prop
-valued class, defined by saying that for every two objects X
and
Y
, the map F.map : (X ⟶ Y) → (F.obj X ⟶ F.obj Y)
is a morphism of abelian groups.
A functor F
is additive provided F.map
is an additive homomorphism.
Instances of this typeclass
- category_theory.functor.id.additive
- category_theory.functor.comp.additive
- category_theory.functor.induced_functor_additive
- category_theory.functor.full_subcategory_inclusion_additive
- category_theory.equivalence.inverse_additive
- category_theory.AdditiveFunctor.forget.functor.additive
- category_theory.AdditiveFunctor.field_1.functor.additive
- category_theory.tensor_left_additive
- category_theory.tensor_right_additive
- category_theory.tensoring_left_additive
- category_theory.tensoring_right_additive
- Action.forget_additive
- Action.forget₂_additive
- Action.functor_category_equivalence_additive
- Action.res_additive
- category_theory.functor.map_Action_preadditive
- Module.forget₂_AddCommGroup_additive
- category_theory.functor.op_additive
- category_theory.functor.right_op_additive
- category_theory.functor.left_op_additive
- category_theory.functor.unop_additive
- category_theory.additive_yoneda_obj
- category_theory.additive_yoneda_obj'
- category_theory.additive_coyoneda_obj
- category_theory.additive_coyoneda_obj'
- category_theory.linear_yoneda_obj_additive
- category_theory.linear_coyoneda_obj_additive
- category_theory.Free.lift_additive
- category_theory.monoidal_category.full_monoidal_subcategory_inclusion_additive
- fgModule.forget₂_monoidal_additive
- homological_complex.eval_additive
- homological_complex.cycles_additive
- homological_complex.boundaries_additive
- homological_complex.homology_additive
- category_theory.functor.map_homogical_complex_additive
- category_theory.idempotents.to_karoubi.category_theory.functor.additive
- category_theory.idempotents.to_karoubi_equivalence_functor_additive
- homological_complex.op_functor_additive
- homological_complex.unop_functor_additive
- category_theory.presheaf_to_Sheaf_additive
- category_theory.idempotents.karoubi_karoubi.inverse.category_theory.functor.additive
- category_theory.idempotents.karoubi_karoubi.equivalence.additive_functor
- category_theory.idempotents.karoubi_karoubi.equivalence.additive_inverse
- category_theory.monad.forget_additive
- category_theory.comonad.forget_additive
- category_theory.Mat_.embedding.category_theory.functor.additive
- category_theory.Mat_.lift_additive
- category_theory.algebra.forget_additive
- category_theory.coalgebra.forget_additive
- SemiNormedGroup.Completion.category_theory.functor.additive
F.map_add_hom
is an additive homomorphism whose underlying function is F.map
.
Equations
- F.map_add_hom = add_monoid_hom.mk' (λ (f : X ⟶ Y), F.map f) _
Equations
- F.preserves_finite_biproducts_of_additive = {preserves := λ (J : Type) (_x : fintype J), {preserves := λ (f : J → C), {preserves := λ (b : category_theory.limits.bicone f) (hb : b.is_bilimit), category_theory.limits.is_bilimit_of_total (F.map_bicone b) _}}}
Bundled additive functors.
Equations
- (C ⥤+ D) = category_theory.full_subcategory (λ (F : C ⥤ D), F.additive)
Instances for category_theory.AdditiveFunctor
An additive functor is in particular a functor.
Equations
- category_theory.AdditiveFunctor.forget C D = category_theory.full_subcategory_inclusion (λ (F : C ⥤ D), F.additive)
Instances for category_theory.AdditiveFunctor.forget
Turn an additive functor into an object of the category AdditiveFunctor C D
.
Equations
- category_theory.AdditiveFunctor.of F = {obj := F, property := _}
Turn a left exact functor into an additive functor.
Equations
Instances for category_theory.AdditiveFunctor.of_left_exact
Turn a right exact functor into an additive functor.
Equations
Instances for category_theory.AdditiveFunctor.of_right_exact
Turn an exact functor into an additive functor.