The short complexes attached to homological complexes #
In this file, we define a functor
shortComplexFunctor C c i : HomologicalComplex C c ⥤ ShortComplex C.
By definition, the image of a homological complex K by this functor
is the short complex K.X (c.prev i) ⟶ K.X i ⟶ K.X (c.next i).
The homology K.homology i of a homological complex K in degree i is defined as
the homology of the short complex (shortComplexFunctor C c i).obj K, which can be
abbreviated as K.sc i.
The functor HomologicalComplex C c ⥤ ShortComplex C which sends a homological
complex K to the short complex K.X i ⟶ K.X j ⟶ K.X k for arbitrary indices i, j and k.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The functor HomologicalComplex C c ⥤ ShortComplex C which sends a homological
complex K to the short complex K.X (c.prev i) ⟶ K.X i ⟶ K.X (c.next i).
Equations
- HomologicalComplex.shortComplexFunctor C c i = HomologicalComplex.shortComplexFunctor' C c (c.prev i) i (c.next i)
Instances For
The natural isomorphism shortComplexFunctor C c j ≅ shortComplexFunctor' C c i j k
when c.prev j = i and c.next j = k.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The short complex K.X i ⟶ K.X j ⟶ K.X k for arbitrary indices i, j and k.
Equations
- K.sc' i j k = (HomologicalComplex.shortComplexFunctor' C c i j k).obj K
Instances For
The short complex K.X (c.prev i) ⟶ K.X i ⟶ K.X (c.next i).
Equations
- K.sc i = (HomologicalComplex.shortComplexFunctor C c i).obj K
Instances For
The canonical isomorphism K.sc j ≅ K.sc' i j k when c.prev j = i and c.next j = k.
Equations
- K.isoSc' i j k hi hk = (HomologicalComplex.natIsoSc' C c i j k hi hk).app K
Instances For
A homological complex K has homology in degree i if the associated
short complex K.sc i has.
Equations
- K.HasHomology i = (K.sc i).HasHomology
Instances For
The homology in degree i of a homological complex.
Instances For
The cycles in degree i of a homological complex.
Instances For
The inclusion of the cycles of a homological complex.
Instances For
The homology class map from cycles to the homology of a homological complex.
Instances For
The morphism to K.cycles i that is induced by a "cycle", i.e. a morphism
to K.X i whose postcomposition with the differential is zero.
Equations
- K.liftCycles k j hj hk = (K.sc i).liftCycles k ⋯
Instances For
The morphism to K.cycles i that is induced by a "cycle", i.e. a morphism
to K.X i whose postcomposition with the differential is zero.
Equations
- K.liftCycles' k j hj hk = K.liftCycles k j ⋯ hk
Instances For
The map K.X i ⟶ K.cycles j induced by the differential K.d i j.
Equations
- K.toCycles i j = K.liftCycles (K.d i j) (c.next j) ⋯ ⋯
Instances For
K.cycles i is the kernel of K.d i j when c.next i = j.
Equations
- K.cyclesIsKernel i j hj = hj ▸ (K.sc i).cyclesIsKernel
Instances For
K.homology j is the cokernel of K.toCycles i j : K.X i ⟶ K.cycles j
when c.prev j = i.
Equations
- K.homologyIsCokernel i j hi = hi ▸ (K.sc j).homologyIsCokernel
Instances For
The opcycles in degree i of a homological complex.
Instances For
The projection to the opcycles of a homological complex.
Instances For
The inclusion map of the homology of a homological complex into its opcycles.
Instances For
The morphism from K.opcycles i that is induced by an "opcycle", i.e. a morphism
from K.X i whose precomposition with the differential is zero.
Equations
- K.descOpcycles k j hj hk = (K.sc i).descOpcycles k ⋯
Instances For
The morphism from K.opcycles i that is induced by an "opcycle", i.e. a morphism
from K.X i whose precomposition with the differential is zero.
Equations
- K.descOpcycles' k j hj hk = K.descOpcycles k j ⋯ hk
Instances For
The map K.opcycles i ⟶ K.X j induced by the differential K.d i j.
Equations
- K.fromOpcycles i j = K.descOpcycles (K.d i j) (c.prev i) ⋯ ⋯
Instances For
K.opcycles j is the cokernel of K.d i j when c.prev j = i.
Equations
- One or more equations did not get rendered due to their size.
Instances For
K.homology i is the kernel of K.fromOpcycles i j : K.opcycles i ⟶ K.X j
when c.next i = j.
Equations
- K.homologyIsKernel i j hi = hi ▸ (K.sc i).homologyIsKernel
Instances For
The map K.homology i ⟶ L.homology i induced by a morphism in HomologicalComplex.
Equations
Instances For
The map K.cycles i ⟶ L.cycles i induced by a morphism in HomologicalComplex.
Equations
Instances For
The map K.opcycles i ⟶ L.opcycles i induced by a morphism in HomologicalComplex.
Equations
Instances For
The isomorphism K.homology i ≅ L.homology i induced by an isomorphism
in HomologicalComplex.
Equations
- HomologicalComplex.homologyMapIso iso i = { hom := HomologicalComplex.homologyMap iso.hom i, inv := HomologicalComplex.homologyMap iso.inv i, hom_inv_id := ⋯, inv_hom_id := ⋯ }
Instances For
The isomorphism K.cycles i ≅ L.cycles i induced by an isomorphism
in HomologicalComplex.
Equations
- HomologicalComplex.cyclesMapIso iso i = { hom := HomologicalComplex.cyclesMap iso.hom i, inv := HomologicalComplex.cyclesMap iso.inv i, hom_inv_id := ⋯, inv_hom_id := ⋯ }
Instances For
The isomorphism K.opcycles i ≅ L.opcycles i induced by an isomorphism
in HomologicalComplex.
Equations
- HomologicalComplex.opcyclesMapIso iso i = { hom := HomologicalComplex.opcyclesMap iso.hom i, inv := HomologicalComplex.opcyclesMap iso.inv i, hom_inv_id := ⋯, inv_hom_id := ⋯ }
Instances For
The ith homology functor HomologicalComplex C c ⥤ C.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The homology functor to graded objects.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The ith cycles functor HomologicalComplex C c ⥤ C.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The ith opcycles functor HomologicalComplex C c ⥤ C.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The natural transformation K.homologyπ i : K.cycles i ⟶ K.homology i
for all K : HomologicalComplex C c.
Equations
- HomologicalComplex.natTransHomologyπ C c i = { app := fun (K : HomologicalComplex C c) => K.homologyπ i, naturality := ⋯ }
Instances For
The natural transformation K.homologyι i : K.homology i ⟶ K.opcycles i
for all K : HomologicalComplex C c.
Equations
- HomologicalComplex.natTransHomologyι C c i = { app := fun (K : HomologicalComplex C c) => K.homologyι i, naturality := ⋯ }
Instances For
The natural isomorphism K.homology i ≅ (K.sc i).homology
for all homological complexes K.
Equations
Instances For
The natural isomorphism K.homology j ≅ (K.sc' i j k).homology
for all homological complexes K when c.prev j = i and c.next j = k.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The canonical isomorphism K.cycles i ≅ K.X i when the differential from i is zero.
Equations
- K.iCyclesIso i j hj h = CategoryTheory.asIso (K.iCycles i)
Instances For
The canonical isomorphism K.homology i ≅ K.opcycles i
when the differential from i is zero.
Equations
- K.isoHomologyι i j hj h = CategoryTheory.asIso (K.homologyι i)
Instances For
The canonical isomorphism K.X j ≅ K.opCycles j when the differential to j is zero.
Equations
- K.pOpcyclesIso i j hi h = CategoryTheory.asIso (K.pOpcycles j)
Instances For
The canonical isomorphism K.cycles j ≅ K.homology j
when the differential to j is zero.
Equations
- K.isoHomologyπ i j hi h = CategoryTheory.asIso (K.homologyπ j)
Instances For
A homological complex K is exact at i if the short complex K.sc i is exact.
Instances For
A homological complex K is acyclic if it is exact at i for any i.
Instances For
The canonical isomorphism K.homology 0 ≅ K.opcycles 0 for a chain complex K
indexed by ℕ.
Equations
Instances For
The canonical isomorphism K.cycles 0 ≅ K.homology 0 for a cochain complex K
indexed by ℕ.
Equations
Instances For
The cycles of a homological complex in degree j can be computed
by specifying a choice of c.prev j and c.next j.
Equations
- K.cyclesIsoSc' i j k hi hk = CategoryTheory.ShortComplex.cyclesMapIso (K.isoSc' i j k hi hk)
Instances For
The homology of a homological complex in degree j can be computed
by specifying a choice of c.prev j and c.next j.
Equations
- K.opcyclesIsoSc' i j k hi hk = CategoryTheory.ShortComplex.opcyclesMapIso (K.isoSc' i j k hi hk)
Instances For
The opcycles of a homological complex in degree j can be computed
by specifying a choice of c.prev j and c.next j.
Equations
- K.homologyIsoSc' i j k hi hk = CategoryTheory.ShortComplex.homologyMapIso (K.isoSc' i j k hi hk)