Documentation

Mathlib.CategoryTheory.MorphismProperty

Properties of morphisms #

We provide the basic framework for talking about properties of morphisms. The following meta-properties are defined

A MorphismProperty C is a class of morphisms between objects in C.

Instances For

    The morphism property in Cᵒᵖ associated to a morphism property in C

    Instances For

      The morphism property in C associated to a morphism property in Cᵒᵖ

      Instances For

        A morphism property RespectsIso if it still holds when composed with an isomorphism

        Instances For

          A morphism property is StableUnderComposition if the composition of two such morphisms still falls in the class.

          Instances For

            A morphism property is StableUnderInverse if the inverse of a morphism satisfying the property still falls in the class.

            Instances For

              A morphism property is StableUnderBaseChange if the base change of such a morphism still falls in the class.

              Instances For

                A morphism property is StableUnderCobaseChange if the cobase change of such a morphism still falls in the class.

                Instances For

                  If P : MorphismProperty C and F : C ⥤ D, then P.IsInvertedBy F means that all morphisms in P are mapped by F to isomorphisms in D.

                  Instances For

                    Given app : Π X, F₁.obj X ⟶ F₂.obj X where F₁ and F₂ are two functors, this is the morphism_property C satisfied by the morphisms in C with respect to whom app is natural.

                    Instances For

                      The full subcategory of C ⥤ D consisting of functors inverting morphisms in W

                      Instances For

                        For P : MorphismProperty C, P.diagonal is a morphism property that holds for f : X ⟶ Y whenever P holds for X ⟶ Y xₓ Y.

                        Instances For

                          P.universally holds for a morphism f : X ⟶ Y iff P holds for all X ×[Y] Y' ⟶ Y'.

                          Instances For
                            theorem CategoryTheory.MorphismProperty.universally_mono {C : Type u} [CategoryTheory.Category.{v, u} C] :
                            Monotone CategoryTheory.MorphismProperty.universally

                            Typeclass expressing that a morphism property contain identities.

                            Instances

                              A morphism property is multiplicative if it contains identities and is stable by composition.

                              Instances