Documentation

Mathlib.AlgebraicTopology.CechNerve

The Čech Nerve #

This file provides a definition of the Čech nerve associated to an arrow, provided the base category has the correct wide pullbacks.

Several variants are provided, given f : Arrow C:

  1. f.cechNerve is the Čech nerve, considered as a simplicial object in C.
  2. f.augmentedCechNerve is the augmented Čech nerve, considered as an augmented simplicial object in C.
  3. SimplicialObject.cechNerve and SimplicialObject.augmentedCechNerve are functorial versions of 1 resp. 2.

We end the file with a description of the Čech nerve of an arrow X ⟶ ⊤_ C to a terminal object, when C has finite products. We call this cechNerveTerminalFrom. When C is G-Set this gives us EG (the universal cover of the classifying space of G) as a simplicial G-set, which is useful for group cohomology.

@[simp]
theorem CategoryTheory.Arrow.cechNerve_obj {C : Type u} [CategoryTheory.Category.{v, u} C] (f : CategoryTheory.Arrow C) [∀ (n : ), CategoryTheory.Limits.HasWidePullback f.right (fun (x : Fin (n + 1)) => f.left) fun (x : Fin (n + 1)) => f.hom] (n : SimplexCategoryᵒᵖ) :
(CategoryTheory.Arrow.cechNerve f).obj n = CategoryTheory.Limits.widePullback f.right (fun (x : Fin (SimplexCategory.len n.unop + 1)) => f.left) fun (x : Fin (SimplexCategory.len n.unop + 1)) => f.hom
@[simp]
def CategoryTheory.Arrow.cechNerve {C : Type u} [CategoryTheory.Category.{v, u} C] (f : CategoryTheory.Arrow C) [∀ (n : ), CategoryTheory.Limits.HasWidePullback f.right (fun (x : Fin (n + 1)) => f.left) fun (x : Fin (n + 1)) => f.hom] :

The Čech nerve associated to an arrow.

Equations
  • One or more equations did not get rendered due to their size.
Instances For
    @[simp]
    theorem CategoryTheory.Arrow.mapCechNerve_app {C : Type u} [CategoryTheory.Category.{v, u} C] {f : CategoryTheory.Arrow C} {g : CategoryTheory.Arrow C} [∀ (n : ), CategoryTheory.Limits.HasWidePullback f.right (fun (x : Fin (n + 1)) => f.left) fun (x : Fin (n + 1)) => f.hom] [∀ (n : ), CategoryTheory.Limits.HasWidePullback g.right (fun (x : Fin (n + 1)) => g.left) fun (x : Fin (n + 1)) => g.hom] (F : f g) (n : SimplexCategoryᵒᵖ) :
    def CategoryTheory.Arrow.mapCechNerve {C : Type u} [CategoryTheory.Category.{v, u} C] {f : CategoryTheory.Arrow C} {g : CategoryTheory.Arrow C} [∀ (n : ), CategoryTheory.Limits.HasWidePullback f.right (fun (x : Fin (n + 1)) => f.left) fun (x : Fin (n + 1)) => f.hom] [∀ (n : ), CategoryTheory.Limits.HasWidePullback g.right (fun (x : Fin (n + 1)) => g.left) fun (x : Fin (n + 1)) => g.hom] (F : f g) :

    The morphism between Čech nerves associated to a morphism of arrows.

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      @[simp]
      theorem CategoryTheory.Arrow.augmentedCechNerve_right {C : Type u} [CategoryTheory.Category.{v, u} C] (f : CategoryTheory.Arrow C) [∀ (n : ), CategoryTheory.Limits.HasWidePullback f.right (fun (x : Fin (n + 1)) => f.left) fun (x : Fin (n + 1)) => f.hom] :

      The augmented Čech nerve associated to an arrow.

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For
        @[simp]
        theorem CategoryTheory.Arrow.mapAugmentedCechNerve_left {C : Type u} [CategoryTheory.Category.{v, u} C] {f : CategoryTheory.Arrow C} {g : CategoryTheory.Arrow C} [∀ (n : ), CategoryTheory.Limits.HasWidePullback f.right (fun (x : Fin (n + 1)) => f.left) fun (x : Fin (n + 1)) => f.hom] [∀ (n : ), CategoryTheory.Limits.HasWidePullback g.right (fun (x : Fin (n + 1)) => g.left) fun (x : Fin (n + 1)) => g.hom] (F : f g) :
        @[simp]
        theorem CategoryTheory.Arrow.mapAugmentedCechNerve_right {C : Type u} [CategoryTheory.Category.{v, u} C] {f : CategoryTheory.Arrow C} {g : CategoryTheory.Arrow C} [∀ (n : ), CategoryTheory.Limits.HasWidePullback f.right (fun (x : Fin (n + 1)) => f.left) fun (x : Fin (n + 1)) => f.hom] [∀ (n : ), CategoryTheory.Limits.HasWidePullback g.right (fun (x : Fin (n + 1)) => g.left) fun (x : Fin (n + 1)) => g.hom] (F : f g) :
        def CategoryTheory.Arrow.mapAugmentedCechNerve {C : Type u} [CategoryTheory.Category.{v, u} C] {f : CategoryTheory.Arrow C} {g : CategoryTheory.Arrow C} [∀ (n : ), CategoryTheory.Limits.HasWidePullback f.right (fun (x : Fin (n + 1)) => f.left) fun (x : Fin (n + 1)) => f.hom] [∀ (n : ), CategoryTheory.Limits.HasWidePullback g.right (fun (x : Fin (n + 1)) => g.left) fun (x : Fin (n + 1)) => g.hom] (F : f g) :

        The morphism between augmented Čech nerve associated to a morphism of arrows.

        Equations
        Instances For
          @[simp]
          theorem CategoryTheory.SimplicialObject.cechNerve_obj {C : Type u} [CategoryTheory.Category.{v, u} C] [∀ (n : ) (f : CategoryTheory.Arrow C), CategoryTheory.Limits.HasWidePullback f.right (fun (x : Fin (n + 1)) => f.left) fun (x : Fin (n + 1)) => f.hom] (f : CategoryTheory.Arrow C) :
          CategoryTheory.SimplicialObject.cechNerve.obj f = CategoryTheory.Arrow.cechNerve f
          @[simp]
          theorem CategoryTheory.SimplicialObject.cechNerve_map {C : Type u} [CategoryTheory.Category.{v, u} C] [∀ (n : ) (f : CategoryTheory.Arrow C), CategoryTheory.Limits.HasWidePullback f.right (fun (x : Fin (n + 1)) => f.left) fun (x : Fin (n + 1)) => f.hom] :
          ∀ {X Y : CategoryTheory.Arrow C} (F : X Y), CategoryTheory.SimplicialObject.cechNerve.map F = CategoryTheory.Arrow.mapCechNerve F

          The Čech nerve construction, as a functor from Arrow C.

          Equations
          • One or more equations did not get rendered due to their size.
          Instances For
            @[simp]
            theorem CategoryTheory.SimplicialObject.augmentedCechNerve_map_right {C : Type u} [CategoryTheory.Category.{v, u} C] [∀ (n : ) (f : CategoryTheory.Arrow C), CategoryTheory.Limits.HasWidePullback f.right (fun (x : Fin (n + 1)) => f.left) fun (x : Fin (n + 1)) => f.hom] :
            ∀ {X Y : CategoryTheory.Arrow C} (F : X Y), (CategoryTheory.SimplicialObject.augmentedCechNerve.map F).right = F.right
            @[simp]
            theorem CategoryTheory.SimplicialObject.augmentedCechNerve_obj_hom_app {C : Type u} [CategoryTheory.Category.{v, u} C] [∀ (n : ) (f : CategoryTheory.Arrow C), CategoryTheory.Limits.HasWidePullback f.right (fun (x : Fin (n + 1)) => f.left) fun (x : Fin (n + 1)) => f.hom] (f : CategoryTheory.Arrow C) (i : SimplexCategoryᵒᵖ) :
            (CategoryTheory.SimplicialObject.augmentedCechNerve.obj f).hom.app i = CategoryTheory.Limits.WidePullback.base fun (x : Fin (SimplexCategory.len i.unop + 1)) => f.hom
            @[simp]
            theorem CategoryTheory.SimplicialObject.augmentedCechNerve_obj_left_map {C : Type u} [CategoryTheory.Category.{v, u} C] [∀ (n : ) (f : CategoryTheory.Arrow C), CategoryTheory.Limits.HasWidePullback f.right (fun (x : Fin (n + 1)) => f.left) fun (x : Fin (n + 1)) => f.hom] (f : CategoryTheory.Arrow C) :
            ∀ {X Y : SimplexCategoryᵒᵖ} (g : X Y), (CategoryTheory.SimplicialObject.augmentedCechNerve.obj f).left.map g = CategoryTheory.Limits.WidePullback.lift (CategoryTheory.Limits.WidePullback.base fun (x : Fin (SimplexCategory.len X.unop + 1)) => f.hom) (fun (i : Fin (SimplexCategory.len Y.unop + 1)) => CategoryTheory.Limits.WidePullback.π (fun (x : Fin (SimplexCategory.len X.unop + 1)) => f.hom) ((SimplexCategory.Hom.toOrderHom g.unop) i))
            @[simp]
            theorem CategoryTheory.SimplicialObject.augmentedCechNerve_obj_left_obj {C : Type u} [CategoryTheory.Category.{v, u} C] [∀ (n : ) (f : CategoryTheory.Arrow C), CategoryTheory.Limits.HasWidePullback f.right (fun (x : Fin (n + 1)) => f.left) fun (x : Fin (n + 1)) => f.hom] (f : CategoryTheory.Arrow C) (n : SimplexCategoryᵒᵖ) :
            (CategoryTheory.SimplicialObject.augmentedCechNerve.obj f).left.obj n = CategoryTheory.Limits.widePullback f.right (fun (x : Fin (SimplexCategory.len n.unop + 1)) => f.left) fun (x : Fin (SimplexCategory.len n.unop + 1)) => f.hom
            @[simp]
            theorem CategoryTheory.SimplicialObject.augmentedCechNerve_obj_right {C : Type u} [CategoryTheory.Category.{v, u} C] [∀ (n : ) (f : CategoryTheory.Arrow C), CategoryTheory.Limits.HasWidePullback f.right (fun (x : Fin (n + 1)) => f.left) fun (x : Fin (n + 1)) => f.hom] (f : CategoryTheory.Arrow C) :
            (CategoryTheory.SimplicialObject.augmentedCechNerve.obj f).right = f.right
            @[simp]
            theorem CategoryTheory.SimplicialObject.augmentedCechNerve_map_left_app {C : Type u} [CategoryTheory.Category.{v, u} C] [∀ (n : ) (f : CategoryTheory.Arrow C), CategoryTheory.Limits.HasWidePullback f.right (fun (x : Fin (n + 1)) => f.left) fun (x : Fin (n + 1)) => f.hom] :
            ∀ {X Y : CategoryTheory.Arrow C} (F : X Y) (n : SimplexCategoryᵒᵖ), (CategoryTheory.SimplicialObject.augmentedCechNerve.map F).left.app n = CategoryTheory.Limits.WidePullback.lift (CategoryTheory.CategoryStruct.comp (CategoryTheory.Limits.WidePullback.base fun (x : Fin (SimplexCategory.len n.unop + 1)) => X.hom) F.right) (fun (i : Fin (SimplexCategory.len n.unop + 1)) => CategoryTheory.CategoryStruct.comp (CategoryTheory.Limits.WidePullback.π (fun (x : Fin (SimplexCategory.len n.unop + 1)) => X.hom) i) F.left)

            The augmented Čech nerve construction, as a functor from Arrow C.

            Equations
            • One or more equations did not get rendered due to their size.
            Instances For
              def CategoryTheory.SimplicialObject.equivalenceRightToLeft {C : Type u} [CategoryTheory.Category.{v, u} C] [∀ (n : ) (f : CategoryTheory.Arrow C), CategoryTheory.Limits.HasWidePullback f.right (fun (x : Fin (n + 1)) => f.left) fun (x : Fin (n + 1)) => f.hom] (X : CategoryTheory.SimplicialObject.Augmented C) (F : CategoryTheory.Arrow C) (G : X CategoryTheory.Arrow.augmentedCechNerve F) :
              CategoryTheory.SimplicialObject.Augmented.toArrow.obj X F

              A helper function used in defining the Čech adjunction.

              Equations
              • One or more equations did not get rendered due to their size.
              Instances For
                @[simp]
                theorem CategoryTheory.SimplicialObject.equivalenceLeftToRight_right {C : Type u} [CategoryTheory.Category.{v, u} C] [∀ (n : ) (f : CategoryTheory.Arrow C), CategoryTheory.Limits.HasWidePullback f.right (fun (x : Fin (n + 1)) => f.left) fun (x : Fin (n + 1)) => f.hom] (X : CategoryTheory.SimplicialObject.Augmented C) (F : CategoryTheory.Arrow C) (G : CategoryTheory.SimplicialObject.Augmented.toArrow.obj X F) :
                @[simp]
                theorem CategoryTheory.SimplicialObject.equivalenceLeftToRight_left_app {C : Type u} [CategoryTheory.Category.{v, u} C] [∀ (n : ) (f : CategoryTheory.Arrow C), CategoryTheory.Limits.HasWidePullback f.right (fun (x : Fin (n + 1)) => f.left) fun (x : Fin (n + 1)) => f.hom] (X : CategoryTheory.SimplicialObject.Augmented C) (F : CategoryTheory.Arrow C) (G : CategoryTheory.SimplicialObject.Augmented.toArrow.obj X F) (x : SimplexCategoryᵒᵖ) :
                def CategoryTheory.SimplicialObject.equivalenceLeftToRight {C : Type u} [CategoryTheory.Category.{v, u} C] [∀ (n : ) (f : CategoryTheory.Arrow C), CategoryTheory.Limits.HasWidePullback f.right (fun (x : Fin (n + 1)) => f.left) fun (x : Fin (n + 1)) => f.hom] (X : CategoryTheory.SimplicialObject.Augmented C) (F : CategoryTheory.Arrow C) (G : CategoryTheory.SimplicialObject.Augmented.toArrow.obj X F) :

                A helper function used in defining the Čech adjunction.

                Equations
                • One or more equations did not get rendered due to their size.
                Instances For
                  @[simp]
                  def CategoryTheory.SimplicialObject.cechNerveEquiv {C : Type u} [CategoryTheory.Category.{v, u} C] [∀ (n : ) (f : CategoryTheory.Arrow C), CategoryTheory.Limits.HasWidePullback f.right (fun (x : Fin (n + 1)) => f.left) fun (x : Fin (n + 1)) => f.hom] (X : CategoryTheory.SimplicialObject.Augmented C) (F : CategoryTheory.Arrow C) :
                  (CategoryTheory.SimplicialObject.Augmented.toArrow.obj X F) (X CategoryTheory.Arrow.augmentedCechNerve F)

                  A helper function used in defining the Čech adjunction.

                  Equations
                  • One or more equations did not get rendered due to their size.
                  Instances For
                    @[inline, reducible]
                    abbrev CategoryTheory.SimplicialObject.cechNerveAdjunction {C : Type u} [CategoryTheory.Category.{v, u} C] [∀ (n : ) (f : CategoryTheory.Arrow C), CategoryTheory.Limits.HasWidePullback f.right (fun (x : Fin (n + 1)) => f.left) fun (x : Fin (n + 1)) => f.hom] :
                    CategoryTheory.SimplicialObject.Augmented.toArrow CategoryTheory.SimplicialObject.augmentedCechNerve

                    The augmented Čech nerve construction is right adjoint to the toArrow functor.

                    Equations
                    • One or more equations did not get rendered due to their size.
                    Instances For
                      @[simp]
                      theorem CategoryTheory.Arrow.cechConerve_obj {C : Type u} [CategoryTheory.Category.{v, u} C] (f : CategoryTheory.Arrow C) [∀ (n : ), CategoryTheory.Limits.HasWidePushout f.left (fun (x : Fin (n + 1)) => f.right) fun (x : Fin (n + 1)) => f.hom] (n : SimplexCategory) :
                      (CategoryTheory.Arrow.cechConerve f).obj n = CategoryTheory.Limits.widePushout f.left (fun (x : Fin (SimplexCategory.len n + 1)) => f.right) fun (x : Fin (SimplexCategory.len n + 1)) => f.hom
                      def CategoryTheory.Arrow.cechConerve {C : Type u} [CategoryTheory.Category.{v, u} C] (f : CategoryTheory.Arrow C) [∀ (n : ), CategoryTheory.Limits.HasWidePushout f.left (fun (x : Fin (n + 1)) => f.right) fun (x : Fin (n + 1)) => f.hom] :

                      The Čech conerve associated to an arrow.

                      Equations
                      • One or more equations did not get rendered due to their size.
                      Instances For
                        @[simp]
                        theorem CategoryTheory.Arrow.mapCechConerve_app {C : Type u} [CategoryTheory.Category.{v, u} C] {f : CategoryTheory.Arrow C} {g : CategoryTheory.Arrow C} [∀ (n : ), CategoryTheory.Limits.HasWidePushout f.left (fun (x : Fin (n + 1)) => f.right) fun (x : Fin (n + 1)) => f.hom] [∀ (n : ), CategoryTheory.Limits.HasWidePushout g.left (fun (x : Fin (n + 1)) => g.right) fun (x : Fin (n + 1)) => g.hom] (F : f g) (n : SimplexCategory) :
                        def CategoryTheory.Arrow.mapCechConerve {C : Type u} [CategoryTheory.Category.{v, u} C] {f : CategoryTheory.Arrow C} {g : CategoryTheory.Arrow C} [∀ (n : ), CategoryTheory.Limits.HasWidePushout f.left (fun (x : Fin (n + 1)) => f.right) fun (x : Fin (n + 1)) => f.hom] [∀ (n : ), CategoryTheory.Limits.HasWidePushout g.left (fun (x : Fin (n + 1)) => g.right) fun (x : Fin (n + 1)) => g.hom] (F : f g) :

                        The morphism between Čech conerves associated to a morphism of arrows.

                        Equations
                        • One or more equations did not get rendered due to their size.
                        Instances For
                          @[simp]
                          theorem CategoryTheory.Arrow.augmentedCechConerve_left {C : Type u} [CategoryTheory.Category.{v, u} C] (f : CategoryTheory.Arrow C) [∀ (n : ), CategoryTheory.Limits.HasWidePushout f.left (fun (x : Fin (n + 1)) => f.right) fun (x : Fin (n + 1)) => f.hom] :

                          The augmented Čech conerve associated to an arrow.

                          Equations
                          • One or more equations did not get rendered due to their size.
                          Instances For
                            @[simp]
                            theorem CategoryTheory.Arrow.mapAugmentedCechConerve_right {C : Type u} [CategoryTheory.Category.{v, u} C] {f : CategoryTheory.Arrow C} {g : CategoryTheory.Arrow C} [∀ (n : ), CategoryTheory.Limits.HasWidePushout f.left (fun (x : Fin (n + 1)) => f.right) fun (x : Fin (n + 1)) => f.hom] [∀ (n : ), CategoryTheory.Limits.HasWidePushout g.left (fun (x : Fin (n + 1)) => g.right) fun (x : Fin (n + 1)) => g.hom] (F : f g) :
                            @[simp]
                            theorem CategoryTheory.Arrow.mapAugmentedCechConerve_left {C : Type u} [CategoryTheory.Category.{v, u} C] {f : CategoryTheory.Arrow C} {g : CategoryTheory.Arrow C} [∀ (n : ), CategoryTheory.Limits.HasWidePushout f.left (fun (x : Fin (n + 1)) => f.right) fun (x : Fin (n + 1)) => f.hom] [∀ (n : ), CategoryTheory.Limits.HasWidePushout g.left (fun (x : Fin (n + 1)) => g.right) fun (x : Fin (n + 1)) => g.hom] (F : f g) :
                            def CategoryTheory.Arrow.mapAugmentedCechConerve {C : Type u} [CategoryTheory.Category.{v, u} C] {f : CategoryTheory.Arrow C} {g : CategoryTheory.Arrow C} [∀ (n : ), CategoryTheory.Limits.HasWidePushout f.left (fun (x : Fin (n + 1)) => f.right) fun (x : Fin (n + 1)) => f.hom] [∀ (n : ), CategoryTheory.Limits.HasWidePushout g.left (fun (x : Fin (n + 1)) => g.right) fun (x : Fin (n + 1)) => g.hom] (F : f g) :

                            The morphism between augmented Čech conerves associated to a morphism of arrows.

                            Equations
                            Instances For
                              @[simp]
                              theorem CategoryTheory.CosimplicialObject.cechConerve_map {C : Type u} [CategoryTheory.Category.{v, u} C] [∀ (n : ) (f : CategoryTheory.Arrow C), CategoryTheory.Limits.HasWidePushout f.left (fun (x : Fin (n + 1)) => f.right) fun (x : Fin (n + 1)) => f.hom] :
                              ∀ {X Y : CategoryTheory.Arrow C} (F : X Y), CategoryTheory.CosimplicialObject.cechConerve.map F = CategoryTheory.Arrow.mapCechConerve F
                              @[simp]
                              theorem CategoryTheory.CosimplicialObject.cechConerve_obj {C : Type u} [CategoryTheory.Category.{v, u} C] [∀ (n : ) (f : CategoryTheory.Arrow C), CategoryTheory.Limits.HasWidePushout f.left (fun (x : Fin (n + 1)) => f.right) fun (x : Fin (n + 1)) => f.hom] (f : CategoryTheory.Arrow C) :
                              CategoryTheory.CosimplicialObject.cechConerve.obj f = CategoryTheory.Arrow.cechConerve f

                              The Čech conerve construction, as a functor from Arrow C.

                              Equations
                              • One or more equations did not get rendered due to their size.
                              Instances For
                                @[simp]
                                theorem CategoryTheory.CosimplicialObject.augmentedCechConerve_obj {C : Type u} [CategoryTheory.Category.{v, u} C] [∀ (n : ) (f : CategoryTheory.Arrow C), CategoryTheory.Limits.HasWidePushout f.left (fun (x : Fin (n + 1)) => f.right) fun (x : Fin (n + 1)) => f.hom] (f : CategoryTheory.Arrow C) :
                                CategoryTheory.CosimplicialObject.augmentedCechConerve.obj f = CategoryTheory.Arrow.augmentedCechConerve f
                                @[simp]
                                theorem CategoryTheory.CosimplicialObject.augmentedCechConerve_map {C : Type u} [CategoryTheory.Category.{v, u} C] [∀ (n : ) (f : CategoryTheory.Arrow C), CategoryTheory.Limits.HasWidePushout f.left (fun (x : Fin (n + 1)) => f.right) fun (x : Fin (n + 1)) => f.hom] :
                                ∀ {X Y : CategoryTheory.Arrow C} (F : X Y), CategoryTheory.CosimplicialObject.augmentedCechConerve.map F = CategoryTheory.Arrow.mapAugmentedCechConerve F

                                The augmented Čech conerve construction, as a functor from Arrow C.

                                Equations
                                • One or more equations did not get rendered due to their size.
                                Instances For
                                  def CategoryTheory.CosimplicialObject.equivalenceLeftToRight {C : Type u} [CategoryTheory.Category.{v, u} C] [∀ (n : ) (f : CategoryTheory.Arrow C), CategoryTheory.Limits.HasWidePushout f.left (fun (x : Fin (n + 1)) => f.right) fun (x : Fin (n + 1)) => f.hom] (F : CategoryTheory.Arrow C) (X : CategoryTheory.CosimplicialObject.Augmented C) (G : CategoryTheory.Arrow.augmentedCechConerve F X) :
                                  F CategoryTheory.CosimplicialObject.Augmented.toArrow.obj X

                                  A helper function used in defining the Čech conerve adjunction.

                                  Equations
                                  • One or more equations did not get rendered due to their size.
                                  Instances For
                                    @[simp]
                                    theorem CategoryTheory.CosimplicialObject.equivalenceRightToLeft_left {C : Type u} [CategoryTheory.Category.{v, u} C] [∀ (n : ) (f : CategoryTheory.Arrow C), CategoryTheory.Limits.HasWidePushout f.left (fun (x : Fin (n + 1)) => f.right) fun (x : Fin (n + 1)) => f.hom] (F : CategoryTheory.Arrow C) (X : CategoryTheory.CosimplicialObject.Augmented C) (G : F CategoryTheory.CosimplicialObject.Augmented.toArrow.obj X) :
                                    @[simp]
                                    def CategoryTheory.CosimplicialObject.equivalenceRightToLeft {C : Type u} [CategoryTheory.Category.{v, u} C] [∀ (n : ) (f : CategoryTheory.Arrow C), CategoryTheory.Limits.HasWidePushout f.left (fun (x : Fin (n + 1)) => f.right) fun (x : Fin (n + 1)) => f.hom] (F : CategoryTheory.Arrow C) (X : CategoryTheory.CosimplicialObject.Augmented C) (G : F CategoryTheory.CosimplicialObject.Augmented.toArrow.obj X) :

                                    A helper function used in defining the Čech conerve adjunction.

                                    Equations
                                    • One or more equations did not get rendered due to their size.
                                    Instances For
                                      def CategoryTheory.CosimplicialObject.cechConerveEquiv {C : Type u} [CategoryTheory.Category.{v, u} C] [∀ (n : ) (f : CategoryTheory.Arrow C), CategoryTheory.Limits.HasWidePushout f.left (fun (x : Fin (n + 1)) => f.right) fun (x : Fin (n + 1)) => f.hom] (F : CategoryTheory.Arrow C) (X : CategoryTheory.CosimplicialObject.Augmented C) :
                                      (CategoryTheory.Arrow.augmentedCechConerve F X) (F CategoryTheory.CosimplicialObject.Augmented.toArrow.obj X)

                                      A helper function used in defining the Čech conerve adjunction.

                                      Equations
                                      • One or more equations did not get rendered due to their size.
                                      Instances For
                                        @[inline, reducible]
                                        abbrev CategoryTheory.CosimplicialObject.cechConerveAdjunction {C : Type u} [CategoryTheory.Category.{v, u} C] [∀ (n : ) (f : CategoryTheory.Arrow C), CategoryTheory.Limits.HasWidePushout f.left (fun (x : Fin (n + 1)) => f.right) fun (x : Fin (n + 1)) => f.hom] :
                                        CategoryTheory.CosimplicialObject.augmentedCechConerve CategoryTheory.CosimplicialObject.Augmented.toArrow

                                        The augmented Čech conerve construction is left adjoint to the toArrow functor.

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

                                          Given an object X : C, the natural simplicial object sending [n] to Xⁿ⁺¹.

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

                                            The product Xᶥ is the vertex of a limit cone on wideCospan ι X.

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

                                              the isomorphism to the product induced by the limit cone wideCospan ι X

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

                                                Given an object X : C, the Čech nerve of the hom to the terminal object X ⟶ ⊤_ C is naturally isomorphic to a simplicial object sending [n] to Xⁿ⁺¹ (when C is G-Set, this is EG, the universal cover of the classifying space of G.

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