Documentation

Mathlib.CategoryTheory.Limits.Shapes.Reflexive

Reflexive coequalizers #

This file deals with reflexive pairs, which are pairs of morphisms with a common section.

A reflexive coequalizer is a coequalizer of such a pair. These kind of 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.

Main definitions #

Main statements #

TODO #

class CategoryTheory.IsReflexivePair {C : Type u} [CategoryTheory.Category.{v, u} C] {A : C} {B : C} (f : A B) (g : A B) :

The pair f g : A ⟶ B is reflexive if there is a morphism B ⟶ A which is a section for both.

Instances
    class CategoryTheory.IsCoreflexivePair {C : Type u} [CategoryTheory.Category.{v, u} C] {A : C} {B : C} (f : A B) (g : A B) :

    The pair f g : A ⟶ B is coreflexive if there is a morphism B ⟶ A which is a retraction for both.

    Instances
      noncomputable def CategoryTheory.commonSection {C : Type u} [CategoryTheory.Category.{v, u} C] {A : C} {B : C} (f : A B) (g : A B) [CategoryTheory.IsReflexivePair f g] :
      B A

      Get the common section for a reflexive pair.

      Equations
      Instances For
        noncomputable def CategoryTheory.commonRetraction {C : Type u} [CategoryTheory.Category.{v, u} C] {A : C} {B : C} (f : A B) (g : A B) [CategoryTheory.IsCoreflexivePair f g] :
        B A

        Get the common retraction for a coreflexive pair.

        Equations
        Instances For
          theorem CategoryTheory.IsKernelPair.isReflexivePair {C : Type u} [CategoryTheory.Category.{v, u} C] {A : C} {B : C} {R : C} {f : R A} {g : R A} {q : A B} (h : CategoryTheory.IsKernelPair q f g) :

          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.

          instance CategoryTheory.instIsReflexivePairMapAppCounitObj {C : Type u} [CategoryTheory.Category.{v, u} C] {D : Type u₂} [CategoryTheory.Category.{v₂, u₂} D] {F : CategoryTheory.Functor C D} {G : CategoryTheory.Functor D C} (adj : F G) (B : D) :
          CategoryTheory.IsReflexivePair (F.map (G.map (adj.counit.app B))) (adj.counit.app (F.obj (G.obj B)))

          For an adjunction F ⊣ G with counit ε, the pair (FGε_B, ε_FGB) is reflexive.

          Equations
          • =

          C has reflexive coequalizers if it has coequalizers for every reflexive pair.

          Instances

            C has coreflexive equalizers if it has equalizers for every coreflexive pair.

            Instances

              The type of objects for the diagram indexing reflexive (co)equalizers

              Instances For
                Equations
                • CategoryTheory.Limits.WalkingReflexivePair.instDecidableEqHom = CategoryTheory.Limits.WalkingReflexivePair.decEqHom✝

                Composition of morphisms in the diagram indexing reflexive (co)equalizers

                Instances For

                  The inclusion functor forgetting the common section

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

                    Bundle the data of a parallel pair along with a common section as a functor out of the walking reflexive pair

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

                      (Noncomputably) bundle the data of a reflexive pair as a functor out of the walking reflexive pair

                      Equations
                      Instances For

                        The natural isomorphism between the diagram obtained by forgetting the reflexion of ofIsReflexivePair f g and the original parallel pair.

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

                          A reflexivePair composed with a functor is isomorphic to the reflexivePair obtained by applying the functor at each map.

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

                            Forgetting the reflexion yields an equivalence between cocones over a bundled reflexive pair and coforks on the underlying parallel pair.

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

                              A reflexive cofork is a colimit cocone if and only if the underlying cofork is.

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

                                The coequalizer of a reflexive pair can be promoted to the colimit of a diagram out of the walking reflexive pair

                                Equations
                                Instances For

                                  A category has coequalizers of reflexive pairs if and only if it has all colimits indexed by the walking reflexive pair.