Idempotent complete categories #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
In this file, we define the notion of idempotent complete categories (also known as Karoubian categories, or pseudoabelian in the case of preadditive categories).
Main definitions #
is_idempotent_complete Cexpresses thatCis idempotent complete, i.e. all idempotents inCsplit. Other characterisations of idempotent completeness are given byis_idempotent_complete_iff_has_equalizer_of_id_and_idempotentandis_idempotent_complete_iff_idempotents_have_kernels.is_idempotent_complete_of_abelianexpresses that abelian categories are idempotent complete.is_idempotent_complete_iff_of_equivalenceexpresses that if two categoriesCandDare equivalent, thenCis idempotent complete iffDis.is_idempotent_complete_iff_oppositeexpresses thatCᵒᵖis idempotent complete iffCis.
References #
- [Stacks: Karoubian categories] https://stacks.math.columbia.edu/tag/09SF
- idempotents_split : ∀ (X : C) (p : X ⟶ X), p ≫ p = p → (∃ (Y : C) (i : Y ⟶ X) (e : X ⟶ Y), i ≫ e = 𝟙 Y ∧ e ≫ i = p)
A category is idempotent complete iff all idempotent endomorphisms p
split as a composition p = e ≫ i with i ≫ e = 𝟙 _
Instances of this typeclass
- category_theory.idempotents.is_idempotent_complete_of_abelian
- category_theory.idempotents.opposite.category_theory.is_idempotent_complete
- category_theory.idempotents.karoubi.category_theory.is_idempotent_complete
- category_theory.idempotents.functor_category_is_idempotent_complete
- category_theory.idempotents.category_theory.simplicial_object.category_theory.is_idempotent_complete
- category_theory.idempotents.category_theory.cosimplicial_object.category_theory.is_idempotent_complete
- category_theory.idempotents.homological_complex.category_theory.is_idempotent_complete
A category is idempotent complete iff for all idempotent endomorphisms, the equalizer of the identity and this idempotent exists.
A preadditive category is pseudoabelian iff all idempotent endomorphisms have a kernel.
An abelian category is idempotent complete.
If C and D are equivalent categories, that C is idempotent complete iff D is.