Documentation

Mathlib.CategoryTheory.Idempotents.Karoubi

The Karoubi envelope of a category #

In this file, we define the Karoubi envelope Karoubi C of a category C.

Main constructions and definitions #

In a preadditive category C, when an object X decomposes as X ≅ P ⨿ Q, one may consider P as a direct factor of X and up to unique isomorphism, it is determined by the obvious idempotent X ⟶ P ⟶ X which is the projection onto P with kernel Q. More generally, one may define a formal direct factor of an object X : C : it consists of an idempotent p : XX which is thought as the "formal image" of p. The type Karoubi C shall be the type of the objects of the karoubi envelope of C. It makes sense for any category C.

  • X : C

    an object of the underlying category

  • p : self.X self.X

    an endomorphism of the object

  • idem : CategoryTheory.CategoryStruct.comp self.p self.p = self.p

    the condition that the given endomorphism is an idempotent

Instances For

    A morphism P ⟶ Q in the category Karoubi C is a morphism in the underlying category C which satisfies a relation, which in the preadditive case, expresses that it induces a map between the corresponding "formal direct factors" and that it vanishes on the complement formal direct factor.

    Instances For

      The category structure on the karoubi envelope of a category.

      Equations

      It is possible to coerce an object of C into an object of Karoubi C. See also the functor toKaroubi.

      Equations

      The obvious fully faithful functor toKaroubi sends an object X : C to the obvious formal direct factor of X given by 𝟙 X.

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For
        Equations
        • CategoryTheory.Idempotents.instAdd = { add := fun (f g : P Q) => { f := f.f + g.f, comm := } }
        Equations
        • CategoryTheory.Idempotents.instNeg = { neg := fun (f : P Q) => { f := -f.f, comm := } }
        Equations
        • CategoryTheory.Idempotents.instZero = { zero := { f := 0, comm := } }

        The map sending f : P ⟶ Q to f.f : P.X ⟶ Q.X is additive.

        Equations
        Instances For
          @[simp]
          theorem CategoryTheory.Idempotents.Karoubi.sum_hom {C : Type u_1} [CategoryTheory.Category.{u_3, u_1} C] [CategoryTheory.Preadditive C] {P : CategoryTheory.Idempotents.Karoubi C} {Q : CategoryTheory.Idempotents.Karoubi C} {α : Type u_2} (s : Finset α) (f : α(P Q)) :
          (Finset.sum s fun (x : α) => f x).f = Finset.sum s fun (x : α) => (f x).f

          The category Karoubi C is preadditive if C is.

          Equations
          • CategoryTheory.Idempotents.instPreadditiveKaroubiInstCategoryKaroubi = { homGroup := fun (P Q : CategoryTheory.Idempotents.Karoubi C) => inferInstance, add_comp := , comp_add := }

          The split mono which appears in the factorisation decompId P.

          Equations
          Instances For

            The split epi which appears in the factorisation decompId P.

            Equations
            Instances For