Documentation

Mathlib.CategoryTheory.MorphismProperty.Concrete

Morphism properties defined in concrete categories #

In this file, we define the class of morphisms MorphismProperty.injective, MorphismProperty.surjective, MorphismProperty.bijective in concrete categories, and show that it is stable under composition and respect isomorphisms.

We introduce type-classes HasSurjectiveInjectiveFactorization and HasFunctorialSurjectiveInjectiveFactorization expressing that in a concrete category C, all morphisms can be factored (resp. factored functorially) as a surjective map followed by an injective map.

def CategoryTheory.MorphismProperty.injective (C : Type u) [Category.{v, u} C] {FC : CCType u_1} {CC : CType u_2} [(X Y : C) → FunLike (FC X Y) (CC X) (CC Y)] [ConcreteCategory C FC] :

Injectiveness (in a concrete category) as a MorphismProperty

Equations
Instances For
    def CategoryTheory.MorphismProperty.surjective (C : Type u) [Category.{v, u} C] {FC : CCType u_1} {CC : CType u_2} [(X Y : C) → FunLike (FC X Y) (CC X) (CC Y)] [ConcreteCategory C FC] :

    Surjectiveness (in a concrete category) as a MorphismProperty

    Equations
    Instances For
      def CategoryTheory.MorphismProperty.bijective (C : Type u) [Category.{v, u} C] {FC : CCType u_1} {CC : CType u_2} [(X Y : C) → FunLike (FC X Y) (CC X) (CC Y)] [ConcreteCategory C FC] :

      Bijectiveness (in a concrete category) as a MorphismProperty

      Equations
      Instances For
        instance CategoryTheory.MorphismProperty.instIsMultiplicativeInjective (C : Type u) [Category.{v, u} C] {FC : CCType u_1} {CC : CType u_2} [(X Y : C) → FunLike (FC X Y) (CC X) (CC Y)] [ConcreteCategory C FC] :
        instance CategoryTheory.MorphismProperty.instIsMultiplicativeSurjective (C : Type u) [Category.{v, u} C] {FC : CCType u_1} {CC : CType u_2} [(X Y : C) → FunLike (FC X Y) (CC X) (CC Y)] [ConcreteCategory C FC] :
        instance CategoryTheory.MorphismProperty.instIsMultiplicativeBijective (C : Type u) [Category.{v, u} C] {FC : CCType u_1} {CC : CType u_2} [(X Y : C) → FunLike (FC X Y) (CC X) (CC Y)] [ConcreteCategory C FC] :
        instance CategoryTheory.MorphismProperty.injective_respectsIso (C : Type u) [Category.{v, u} C] {FC : CCType u_1} {CC : CType u_2} [(X Y : C) → FunLike (FC X Y) (CC X) (CC Y)] [ConcreteCategory C FC] :
        instance CategoryTheory.MorphismProperty.surjective_respectsIso (C : Type u) [Category.{v, u} C] {FC : CCType u_1} {CC : CType u_2} [(X Y : C) → FunLike (FC X Y) (CC X) (CC Y)] [ConcreteCategory C FC] :
        instance CategoryTheory.MorphismProperty.bijective_respectsIso (C : Type u) [Category.{v, u} C] {FC : CCType u_1} {CC : CType u_2} [(X Y : C) → FunLike (FC X Y) (CC X) (CC Y)] [ConcreteCategory C FC] :
        @[reducible, inline]
        abbrev CategoryTheory.ConcreteCategory.HasSurjectiveInjectiveFactorization (C : Type u) [Category.{v, u} C] {FC : CCType u_1} {CC : CType u_2} [(X Y : C) → FunLike (FC X Y) (CC X) (CC Y)] [ConcreteCategory C FC] :

        The property that any morphism in a concrete category can be factored as a surjective map followed by an injective map.

        Equations
        Instances For
          @[reducible, inline]
          abbrev CategoryTheory.ConcreteCategory.HasFunctorialSurjectiveInjectiveFactorization (C : Type u) [Category.{v, u} C] {FC : CCType u_1} {CC : CType u_2} [(X Y : C) → FunLike (FC X Y) (CC X) (CC Y)] [ConcreteCategory C FC] :

          The property that any morphism in a concrete category can be functorially factored as a surjective map followed by an injective map.

          Equations
          • One or more equations did not get rendered due to their size.
          Instances For
            @[reducible, inline]
            abbrev CategoryTheory.ConcreteCategory.FunctorialSurjectiveInjectiveFactorizationData (C : Type u) [Category.{v, u} C] {FC : CCType u_1} {CC : CType u_2} [(X Y : C) → FunLike (FC X Y) (CC X) (CC Y)] [ConcreteCategory C FC] :
            Type (max u v)

            The structure containing the data of a functorial factorization of morphisms as a surjective map followed by an injective map in a concrete category.

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

              In the category of types, any map can be functorially factored as a surjective map followed by an injective map.

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