Documentation

Mathlib.CategoryTheory.Limits.Shapes.Preorder.TransfiniteCompositionOfShape

A structure to describe transfinite compositions #

Given a well-ordered type J and a morphism f : X ⟶ Y in a category, we introduce a structure TransfiniteCompositionOfShape J f expressing that f is a transfinite composition of shape J. This allows to extend this structure in order to require more properties or data for the morphisms F.obj j ⟶ F.obj (Order.succ j) which appear in the transfinite composition. See MorphismProperty.TransfiniteCompositionOfShape in the file MorphismProperty.TransfiniteComposition.

structure CategoryTheory.TransfiniteCompositionOfShape {C : Type u} [Category.{v, u} C] (J : Type w) [LinearOrder J] [OrderBot J] {X Y : C} (f : X Y) [SuccOrder J] [WellFoundedLT J] :
Type (max (max u v) w)

Given a well-ordered type J, a morphism f : X ⟶ Y in a category C is a transfinite composition of shape J if we have a well order continuous functor F : J ⥤ C, an isomorphism F.obj ⊥ ≅ X, a colimit cocone for F whose point is Y, such that the composition X ⟶ F.obj ⊥ ⟶ Y is f.

Instances For

    If f and f' are two isomorphic morphisms, and f is a transfinite composition of shape J, then f' also is.

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      @[simp]
      theorem CategoryTheory.TransfiniteCompositionOfShape.ofArrowIso_F {C : Type u} [Category.{v, u} C] {J : Type w} [LinearOrder J] [OrderBot J] {X Y : C} {f : X Y} [SuccOrder J] [WellFoundedLT J] (c : TransfiniteCompositionOfShape J f) {X' Y' : C} {f' : X' Y'} (e : Arrow.mk f Arrow.mk f') :
      (c.ofArrowIso e).F = c.F

      If G : ComposableArrows C n, then G.hom : G.left ⟶ G.right is a transfinite composition of shape Fin (n + 1).

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

        If f is a transfinite composition of shape J, then it is also a transfinite composition of shape J' if J' ≃o J.

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

          If f is a transfinite composition of shape J, then F.map f also is provided F preserves suitable colimits.

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

            A transfinite composition of shape J induces a transfinite composition of shape Set.Iic j for any j : J.

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