Documentation

Mathlib.AlgebraicTopology.SimplicialObject.Coskeletal

Coskeletal simplicial objects #

The identity natural transformation exhibits a simplicial object X as a right extension of its restriction along (Truncated.inclusion n).op recorded by rightExtensionInclusion X n.

The simplicial object X is n-coskeletal if rightExtensionInclusion X n is a right Kan extension.

When the ambient category admits right Kan extensions along (Truncated.inclusion n).op, then when X is n-coskeletal, the unit of coskAdj n defines an isomorphism: isoCoskOfIsCoskeletal : X ≅ (cosk n).obj X.

TODO: Prove that X is n-coskeletal whenever a certain canonical cone is a limit cone.

The identity natural transformation exhibits a simplicial set as a right extension of its restriction along (Truncated.inclusion n).op.

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

    A simplicial object X is n-coskeletal when it is the right Kan extension of its restriction along (Truncated.inclusion n).op via the identity natural transformation.

    Instances

      If X is n-coskeletal, then Truncated.rightExtensionInclusion X n is a terminal object in the category RightExtension (Truncated.inclusion n).op (Truncated.inclusion.op ⋙ X).

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For
        theorem CategoryTheory.SimplicialObject.isCoskeletal_iff_isIso {C : Type u} [Category.{v, u} C] (X : SimplicialObject C) (n : ) [∀ (F : Functor (SimplexCategory.Truncated n)ᵒᵖ C), (SimplexCategory.Truncated.inclusion n).op.HasRightKanExtension F] :
        X.IsCoskeletal n IsIso ((coskAdj n).unit.app X)
        instance CategoryTheory.SimplicialObject.instIsIsoAppUnitTruncatedCoskAdj {C : Type u} [Category.{v, u} C] (X : SimplicialObject C) (n : ) [∀ (F : Functor (SimplexCategory.Truncated n)ᵒᵖ C), (SimplexCategory.Truncated.inclusion n).op.HasRightKanExtension F] [X.IsCoskeletal n] :
        IsIso ((coskAdj n).unit.app X)
        noncomputable def CategoryTheory.SimplicialObject.isoCoskOfIsCoskeletal {C : Type u} [Category.{v, u} C] (X : SimplicialObject C) (n : ) [∀ (F : Functor (SimplexCategory.Truncated n)ᵒᵖ C), (SimplexCategory.Truncated.inclusion n).op.HasRightKanExtension F] [X.IsCoskeletal n] :
        X (cosk n).obj X

        The canonical isomorphism X ≅ (cosk n).obj X defined when X is coskeletal and the n-coskeleton functor exists.

        Equations
        Instances For
          @[simp]
          theorem CategoryTheory.SimplicialObject.isoCoskOfIsCoskeletal_hom {C : Type u} [Category.{v, u} C] (X : SimplicialObject C) (n : ) [∀ (F : Functor (SimplexCategory.Truncated n)ᵒᵖ C), (SimplexCategory.Truncated.inclusion n).op.HasRightKanExtension F] [X.IsCoskeletal n] :
          (X.isoCoskOfIsCoskeletal n).hom = (coskAdj n).unit.app X