Documentation

Mathlib.CategoryTheory.Limits.Constructions.Over.Products

Products in the over category #

Shows that products in the over category can be derived from wide pullbacks in the base category. The main result is over_product_of_widePullback, which says that if C has J-indexed wide pullbacks, then Over B has J-indexed products.

@[reducible, inline]

(Implementation) Given a product diagram in C/B, construct the corresponding wide pullback diagram in C.

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

    (Impl) A preliminary definition to avoid timeouts.

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

      (Impl) A preliminary definition to avoid timeouts.

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For
        @[simp]
        theorem CategoryTheory.Over.ConstructProducts.conesEquivInverse_map_hom {C : Type u} [Category.{v, u} C] (B : C) {J : Type w} (F : Functor (Discrete J) (Over B)) {X✝ Y✝ : Limits.Cone F} (f : X✝ Y✝) :

        (Impl) A preliminary definition to avoid timeouts.

        Equations
        • One or more equations did not get rendered due to their size.
        Instances For
          @[simp]
          theorem CategoryTheory.Over.ConstructProducts.conesEquivFunctor_obj_π_app {C : Type u} [Category.{v, u} C] (B : C) {J : Type w} (F : Functor (Discrete J) (Over B)) (c : Limits.Cone (widePullbackDiagramOfDiagramOver B F)) (x✝ : Discrete J) :
          ((conesEquivFunctor B F).obj c).π.app x✝ = match x✝ with | { as := j } => homMk (c.π.app (some j))
          @[simp]

          (Impl) A preliminary definition to avoid timeouts.

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

            (Impl) A preliminary definition to avoid timeouts.

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

              (Impl) Establish an equivalence between the category of cones for F and for the "grown" F.

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

                Given a pullback in C, construct a binary product in C/B.

                Given all wide pullbacks in C, construct products in C/B.

                Given all finite wide pullbacks in C, construct finite products in C/B.

                Construct terminal object in the over category. This isn't an instance as it's not typically the way we want to define terminal objects. (For instance, this gives a terminal object which is different from the generic one given by over_product_of_widePullback above.)

                The product of Y and Z in Over X is isomorpic to Y ×ₓ Z.

                Equations
                Instances For