Homology is an additive functor #
When V
is preadditive, HomologicalComplex V c
is also preadditive,
and homologyFunctor
is additive.
Equations
- HomologicalComplex.instZeroHom_1 = { zero := { f := fun (x : ι) => 0, comm' := ⋯ } }
Equations
- HomologicalComplex.instAddCommGroupHom = Function.Injective.addCommGroup HomologicalComplex.Hom.f ⋯ ⋯ ⋯ ⋯ ⋯ ⋯ ⋯
Equations
- HomologicalComplex.instPreadditive = { homGroup := inferInstance, add_comp := ⋯, comp_add := ⋯ }
The i
-th component of a chain map, as an additive map from chain maps to morphisms.
Equations
- HomologicalComplex.Hom.fAddMonoidHom i = AddMonoidHom.mk' (fun (f : C₁ ⟶ C₂) => f.f i) ⋯
Instances For
An additive functor induces a functor between homological complexes. This is sometimes called the "prolongation".
Equations
- One or more equations did not get rendered due to their size.
Instances For
The functor on homological complexes induced by the identity functor is isomorphic to the identity functor.
Equations
- One or more equations did not get rendered due to their size.
Instances For
A natural transformation between functors induces a natural transformation between those functors applied to homological complexes.
Equations
- CategoryTheory.NatTrans.mapHomologicalComplex α c = { app := fun (C : HomologicalComplex W₁ c) => { f := fun (x : ι) => α.app (C.X x), comm' := ⋯ }, naturality := ⋯ }
Instances For
A natural isomorphism between functors induces a natural isomorphism between those functors applied to homological complexes.
Equations
- One or more equations did not get rendered due to their size.
Instances For
An equivalence of categories induces an equivalences between the respective categories of homological complex.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Turning an object into a complex supported at j
then applying a functor is
the same as applying the functor then forming the complex.
Equations
- One or more equations did not get rendered due to their size.