Documentation

Mathlib.Algebra.Homology.ShortComplex.Exact

Exact short complexes #

When S : ShortComplex C, this file defines a structure S.Exact which expresses the exactness of S, i.e. there exists a homology data h : S.HomologyData such that h.left.H is zero. When [S.HasHomology], it is equivalent to the assertion IsZero S.homology.

Almost by construction, this notion of exactness is self dual, see Exact.op and Exact.unop.

The assertion that the short complex S : ShortComplex C is exact.

Instances For
    theorem CategoryTheory.ShortComplex.exact_of_iso {C : Type u_1} [Category.{u_3, u_1} C] [Limits.HasZeroMorphisms C] {S₁ S₂ : ShortComplex C} (e : S₁ S₂) (h : S₁.Exact) :
    S₂.Exact

    Given an exact short complex S and a limit kernel fork kf for S.g, this is the left homology data for S with K := kf.pt and H := 0.

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For

      Given an exact short complex S and a colimit cokernel cofork cc for S.f, this is the right homology data for S with Q := cc.pt and H := 0.

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For
        theorem CategoryTheory.ShortComplex.QuasiIso.exact_iff {C : Type u_1} [Category.{u_3, u_1} C] [Preadditive C] {S₁ S₂ : ShortComplex C} (φ : S₁ S₂) [S₁.HasHomology] [S₂.HasHomology] [QuasiIso φ] :
        S₁.Exact S₂.Exact

        A splitting for a short complex S consists of the data of a retraction r : X₂ ⟶ X₁ of S.f and section s : X₃ ⟶ X₂ of S.g which satisfy r ≫ S.f + S.g ≫ s = 𝟙 _

        Instances For

          Given a splitting of a short complex S, this shows that S.f is a split monomorphism.

          Equations
          Instances For

            Given a splitting of a short complex S, this shows that S.g is a split epimorphism.

            Equations
            Instances For

              The left homology data on a short complex equipped with a splitting.

              Equations
              • One or more equations did not get rendered due to their size.
              Instances For

                The right homology data on a short complex equipped with a splitting.

                Equations
                • One or more equations did not get rendered due to their size.
                Instances For

                  The homology data on a short complex equipped with a splitting.

                  Equations
                  Instances For

                    A short complex equipped with a splitting is exact.

                    If a short complex S is equipped with a splitting, then S.X₁ is the kernel of S.g.

                    Equations
                    Instances For

                      If a short complex S is equipped with a splitting, then S.X₃ is the cokernel of S.f.

                      Equations
                      Instances For

                        If a short complex S has a splitting and F is an additive functor, then S.map F also has a splitting.

                        Equations
                        • s.map F = { r := F.map s.r, s := F.map s.s, f_r := , s_g := , id := }
                        Instances For
                          @[simp]
                          @[simp]
                          def CategoryTheory.ShortComplex.Splitting.ofIso {C : Type u_1} [Category.{u_3, u_1} C] [Preadditive C] {S₁ S₂ : ShortComplex C} (s : S₁.Splitting) (e : S₁ S₂) :

                          A splitting on a short complex induces splittings on isomorphic short complexes.

                          Equations
                          • One or more equations did not get rendered due to their size.
                          Instances For

                            The obvious splitting of the short complex X₁ ⟶ X₁ ⊞ X₂ ⟶ X₂.

                            Equations
                            Instances For

                              The obvious splitting of a short complex when S.X₁ is zero and S.g is an isomorphism.

                              Equations
                              Instances For

                                The obvious splitting of a short complex when S.f is an isomorphism and S.X₃ is zero.

                                Equations
                                Instances For

                                  The splitting of the short complex S.op deduced from a splitting of S.

                                  Equations
                                  • h.op = { r := h.s.op, s := h.r.op, f_r := , s_g := , id := }
                                  Instances For

                                    The splitting of the short complex S.unop deduced from a splitting of S.

                                    Equations
                                    • h.unop = { r := h.s.unop, s := h.r.unop, f_r := , s_g := , id := }
                                    Instances For

                                      The isomorphism S.X₂ ≅ S.X₁ ⊞ S.X₃ induced by a splitting of the short complex S.

                                      Equations
                                      Instances For

                                        In a balanced category, if a short complex S is exact and S.f is a mono, then S.X₁ is the kernel of S.g.

                                        Equations
                                        Instances For

                                          In a balanced category, if a short complex S is exact and S.g is an epi, then S.X₃ is the cokernel of S.g.

                                          Equations
                                          Instances For
                                            noncomputable def CategoryTheory.ShortComplex.Exact.lift {C : Type u_1} [Category.{u_3, u_1} C] [Preadditive C] {S : ShortComplex C} [Balanced C] (hS : S.Exact) {A : C} (k : A S.X₂) (hk : CategoryStruct.comp k S.g = 0) [Mono S.f] :
                                            A S.X₁

                                            If a short complex S in a balanced category is exact and such that S.f is a mono, then a morphism k : A ⟶ S.X₂ such that k ≫ S.g = 0 lifts to a morphism A ⟶ S.X₁.

                                            Equations
                                            Instances For
                                              @[simp]
                                              theorem CategoryTheory.ShortComplex.Exact.lift_f {C : Type u_1} [Category.{u_3, u_1} C] [Preadditive C] {S : ShortComplex C} [Balanced C] (hS : S.Exact) {A : C} (k : A S.X₂) (hk : CategoryStruct.comp k S.g = 0) [Mono S.f] :
                                              CategoryStruct.comp (hS.lift k hk) S.f = k
                                              @[simp]
                                              theorem CategoryTheory.ShortComplex.Exact.lift_f_assoc {C : Type u_1} [Category.{u_3, u_1} C] [Preadditive C] {S : ShortComplex C} [Balanced C] (hS : S.Exact) {A : C} (k : A S.X₂) (hk : CategoryStruct.comp k S.g = 0) [Mono S.f] {Z : C} (h : S.X₂ Z) :
                                              theorem CategoryTheory.ShortComplex.Exact.lift' {C : Type u_1} [Category.{u_3, u_1} C] [Preadditive C] {S : ShortComplex C} [Balanced C] (hS : S.Exact) {A : C} (k : A S.X₂) (hk : CategoryStruct.comp k S.g = 0) [Mono S.f] :
                                              ∃ (l : A S.X₁), CategoryStruct.comp l S.f = k
                                              noncomputable def CategoryTheory.ShortComplex.Exact.desc {C : Type u_1} [Category.{u_3, u_1} C] [Preadditive C] {S : ShortComplex C} [Balanced C] (hS : S.Exact) {A : C} (k : S.X₂ A) (hk : CategoryStruct.comp S.f k = 0) [Epi S.g] :
                                              S.X₃ A

                                              If a short complex S in a balanced category is exact and such that S.g is an epi, then a morphism k : S.X₂ ⟶ A such that S.f ≫ k = 0 descends to a morphism S.X₃ ⟶ A.

                                              Equations
                                              Instances For
                                                @[simp]
                                                theorem CategoryTheory.ShortComplex.Exact.g_desc {C : Type u_1} [Category.{u_3, u_1} C] [Preadditive C] {S : ShortComplex C} [Balanced C] (hS : S.Exact) {A : C} (k : S.X₂ A) (hk : CategoryStruct.comp S.f k = 0) [Epi S.g] :
                                                CategoryStruct.comp S.g (hS.desc k hk) = k
                                                @[simp]
                                                theorem CategoryTheory.ShortComplex.Exact.g_desc_assoc {C : Type u_1} [Category.{u_3, u_1} C] [Preadditive C] {S : ShortComplex C} [Balanced C] (hS : S.Exact) {A : C} (k : S.X₂ A) (hk : CategoryStruct.comp S.f k = 0) [Epi S.g] {Z : C} (h : A Z) :
                                                theorem CategoryTheory.ShortComplex.Exact.desc' {C : Type u_1} [Category.{u_3, u_1} C] [Preadditive C] {S : ShortComplex C} [Balanced C] (hS : S.Exact) {A : C} (k : S.X₂ A) (hk : CategoryStruct.comp S.f k = 0) [Epi S.g] :
                                                ∃ (l : S.X₃ A), CategoryStruct.comp S.g l = k
                                                theorem CategoryTheory.ShortComplex.mono_τ₂_of_exact_of_mono {C : Type u_1} [Category.{u_3, u_1} C] [Preadditive C] [Balanced C] {S₁ S₂ : ShortComplex C} (φ : S₁ S₂) (h₁ : S₁.Exact) [Mono S₁.f] [Mono S₂.f] [Mono φ.τ₁] [Mono φ.τ₃] :
                                                theorem CategoryTheory.ShortComplex.epi_τ₂_of_exact_of_epi {C : Type u_1} [Category.{u_3, u_1} C] [Preadditive C] [Balanced C] {S₁ S₂ : ShortComplex C} (φ : S₁ S₂) (h₂ : S₂.Exact) [Epi S₁.g] [Epi S₂.g] [Epi φ.τ₁] [Epi φ.τ₃] :
                                                theorem CategoryTheory.ShortComplex.quasiIso_iff_of_zeros {C : Type u_1} [Category.{u_3, u_1} C] [Abelian C] {S₁ S₂ : ShortComplex C} (φ : S₁ S₂) (hf₁ : S₁.f = 0) (hg₁ : S₁.g = 0) (hf₂ : S₂.f = 0) :
                                                QuasiIso φ (mk φ.τ₂ S₂.g ).Exact Mono φ.τ₂

                                                Given a morphism of short complexes φ : S₁ ⟶ S₂ in an abelian category, if S₁.f and S₁.g are zero (e.g. when S₁ is of the form 0 ⟶ S₁.X₂ ⟶ 0) and S₂.f = 0 (e.g when S₂ is of the form 0 ⟶ S₂.X₂ ⟶ S₂.X₃), then φ is a quasi-isomorphism iff the obvious short complex S₁.X₂ ⟶ S₂.X₂ ⟶ S₂.X₃ is exact and φ.τ₂ is a mono).

                                                theorem CategoryTheory.ShortComplex.quasiIso_iff_of_zeros' {C : Type u_1} [Category.{u_3, u_1} C] [Abelian C] {S₁ S₂ : ShortComplex C} (φ : S₁ S₂) (hg₁ : S₁.g = 0) (hf₂ : S₂.f = 0) (hg₂ : S₂.g = 0) :
                                                QuasiIso φ (mk S₁.f φ.τ₂ ).Exact Epi φ.τ₂

                                                Given a morphism of short complexes φ : S₁ ⟶ S₂ in an abelian category, if S₁.g = 0 (e.g when S₁ is of the form S₁.X₁ ⟶ S₁.X₂ ⟶ 0) and both S₂.f and S₂.g are zero (e.g when S₂ is of the form 0 ⟶ S₂.X₂ ⟶ 0), then φ is a quasi-isomorphism iff the obvious short complex S₁.X₂ ⟶ S₁.X₂ ⟶ S₂.X₂ is exact and φ.τ₂ is an epi).

                                                noncomputable def CategoryTheory.ShortComplex.Exact.descToInjective {C : Type u_1} [Category.{u_3, u_1} C] [Abelian C] {S : ShortComplex C} (hS : S.Exact) {J : C} (f : S.X₂ J) [Injective J] (hf : CategoryStruct.comp S.f f = 0) :
                                                S.X₃ J

                                                If S is an exact short complex and f : S.X₂ ⟶ J is a morphism to an injective object J such that S.f ≫ f = 0, this is a morphism φ : S.X₃ ⟶ J such that S.g ≫ φ = f.

                                                Equations
                                                Instances For
                                                  noncomputable def CategoryTheory.ShortComplex.Exact.liftFromProjective {C : Type u_1} [Category.{u_3, u_1} C] [Abelian C] {S : ShortComplex C} (hS : S.Exact) {P : C} (f : P S.X₂) [Projective P] (hf : CategoryStruct.comp f S.g = 0) :
                                                  P S.X₁

                                                  If S is an exact short complex and f : P ⟶ S.X₂ is a morphism from a projective object P such that f ≫ S.g = 0, this is a morphism φ : P ⟶ S.X₁ such that φ ≫ S.f = f.

                                                  Equations
                                                  Instances For

                                                    This is the splitting of a short complex S in a balanced category induced by a section of the morphism S.g : S.X₂ ⟶ S.X₃

                                                    Equations
                                                    • One or more equations did not get rendered due to their size.
                                                    Instances For

                                                      This is the splitting of a short complex S in a balanced category induced by a retraction of the morphism S.f : S.X₁ ⟶ S.X₂

                                                      Equations
                                                      • One or more equations did not get rendered due to their size.
                                                      Instances For