Reflexive coequalizers #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
We define reflexive pairs as a pair of morphisms which have a common section. We say a category has reflexive coequalizers if it has coequalizers of all reflexive pairs. Reflexive coequalizers often enjoy nicer properties than general coequalizers, and feature heavily in some versions of the monadicity theorem.
We also give some examples of reflexive pairs: for an adjunction F ⊣ G
with counit ε
, the pair
(FGε_B, ε_FGB)
is reflexive. If a pair f,g
is a kernel pair for some morphism, then it is
reflexive.
TODO #
- If
C
has binary coproducts and reflexive coequalizers, then it has all coequalizers. - If
T
is a monad on cocomplete categoryC
, thenalgebra T
is cocomplete iff it has reflexive coequalizers. - If
C
is locally cartesian closed and has reflexive coequalizers, then it has images: in fact regular epi (and hence strong epi) images.
The pair f g : A ⟶ B
is reflexive if there is a morphism B ⟶ A
which is a section for both.
Get the common section for a reflexive pair.
Equations
Get the common retraction for a coreflexive pair.
Equations
If f,g
is a kernel pair for some morphism q
, then it is reflexive.
If f,g
is reflexive, then g,f
is reflexive.
If f,g
is coreflexive, then g,f
is coreflexive.
For an adjunction F ⊣ G
with counit ε
, the pair (FGε_B, ε_FGB)
is reflexive.
- has_coeq : ∀ ⦃A B : C⦄ (f g : A ⟶ B) [_inst_3 : category_theory.is_reflexive_pair f g], category_theory.limits.has_coequalizer f g
C
has reflexive coequalizers if it has coequalizers for every reflexive pair.
Instances of this typeclass
- has_eq : ∀ ⦃A B : C⦄ (f g : A ⟶ B) [_inst_3 : category_theory.is_coreflexive_pair f g], category_theory.limits.has_equalizer f g
C
has coreflexive equalizers if it has equalizers for every coreflexive pair.
Instances of this typeclass
If C
has coequalizers, then it has reflexive coequalizers.
If C
has equalizers, then it has coreflexive equalizers.