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.

Equations
Instances For
    Equations
    • CategoryTheory.MorphismProperty.instHasSubsetMorphismProperty = { Subset := fun (P₁ P₂ : CategoryTheory.MorphismProperty C) => ∀ ⦃X Y : C⦄ (f : X Y), P₁ fP₂ f }
    Equations

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

    Equations
    Instances For

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

      Equations
      Instances For

        The image (up to isomorphisms) of a MorphismProperty C by a functor C ⥤ D

        Equations
        Instances For

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

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

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

            Equations
            Instances For

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

              Equations
              Instances For

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

                Equations
                Instances For

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

                  Equations
                  Instances For
                    theorem CategoryTheory.MorphismProperty.StableUnderBaseChange.pullback_map {C : Type u} [CategoryTheory.Category.{v, u} C] [CategoryTheory.Limits.HasPullbacks C] {P : CategoryTheory.MorphismProperty C} (hP : CategoryTheory.MorphismProperty.StableUnderBaseChange P) (hP' : CategoryTheory.MorphismProperty.StableUnderComposition P) {S : C} {X : C} {X' : C} {Y : C} {Y' : C} {f : X S} {g : Y S} {f' : X' S} {g' : Y' S} {i₁ : X X'} {i₂ : Y Y'} (h₁ : P i₁) (h₂ : P i₂) (e₁ : f = CategoryTheory.CategoryStruct.comp i₁ f') (e₂ : g = CategoryTheory.CategoryStruct.comp i₂ g') :

                    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.

                    Equations
                    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.

                      Equations
                      Instances For

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

                        Equations
                        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

                              If W₁ and W₂ are morphism properties on two categories C₁ and C₂, this is the induced morphism property on C₁ × C₂.

                              Equations
                              Instances For
                                def CategoryTheory.MorphismProperty.pi {J : Type w} {C : JType u} [(j : J) → CategoryTheory.Category.{v, u} (C j)] (W : (j : J) → CategoryTheory.MorphismProperty (C j)) :

                                If W j are morphism properties on categories C j for all j, this is the induced morphism property on the category ∀ j, C j.

                                Equations
                                Instances For

                                  The property that a morphism property W is stable under limits indexed by a category J.

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

                                    The condition that a property of morphisms is stable by finite products.

                                    Instances