Documentation

Mathlib.Topology.Category.CompHaus.Limits

Explicit limits and colimits #

This file collects some constructions of explicit limits and colimits in CompHaus, which may be useful due to their definitional properties.

So far, we have the following:

def CompHaus.pullback {X : CompHaus} {Y : CompHaus} {B : CompHaus} (f : X B) (g : Y B) :

The pullback of two morphisms f,g in CompHaus, constructed explicitly as the set of pairs (x,y) such that f x = g y, with the topology induced by the product.

Equations
Instances For
    def CompHaus.pullback.fst {X : CompHaus} {Y : CompHaus} {B : CompHaus} (f : X B) (g : Y B) :

    The projection from the pullback to the first component.

    Equations
    Instances For
      def CompHaus.pullback.snd {X : CompHaus} {Y : CompHaus} {B : CompHaus} (f : X B) (g : Y B) :

      The projection from the pullback to the second component.

      Equations
      Instances For

        Construct a morphism to the explicit pullback given morphisms to the factors which are compatible with the maps to the base. This is essentially the universal property of the pullback.

        Equations
        • CompHaus.pullback.lift f g a b w = { toFun := fun (z : Z.toTop) => { val := (a z, b z), property := }, continuous_toFun := }
        Instances For
          @[simp]
          theorem CompHaus.pullback.cone_pt {X : CompHaus} {Y : CompHaus} {B : CompHaus} (f : X B) (g : Y B) :

          The pullback cone whose cone point is the explicit pullback.

          Equations
          Instances For

            The explicit pullback cone is a limit cone.

            Equations
            • One or more equations did not get rendered due to their size.
            Instances For
              noncomputable def CompHaus.pullbackHomeoPullback {X : CompHaus} {Y : CompHaus} {B : CompHaus} (f : X B) (g : Y B) :

              The homeomorphism from the explicit pullback to the abstract pullback.

              Equations
              Instances For
                theorem CompHaus.pullback_fst_eq {X : CompHaus} {Y : CompHaus} {B : CompHaus} (f : X B) (g : Y B) :
                theorem CompHaus.pullback_snd_eq {X : CompHaus} {Y : CompHaus} {B : CompHaus} (f : X B) (g : Y B) :
                def CompHaus.finiteCoproduct {α : Type w} [Finite α] (X : αCompHausMax) :

                The coproduct of a finite family of objects in CompHaus, constructed as the disjoint union with its usual topology.

                Equations
                Instances For
                  def CompHaus.finiteCoproduct.ι {α : Type w} [Finite α] (X : αCompHausMax) (a : α) :

                  The inclusion of one of the factors into the explicit finite coproduct.

                  Equations
                  Instances For
                    def CompHaus.finiteCoproduct.desc {α : Type w} [Finite α] (X : αCompHausMax) {B : CompHausMax} (e : (a : α) → X a B) :

                    To construct a morphism from the explicit finite coproduct, it suffices to specify a morphism from each of its factors. This is essentially the universal property of the coproduct.

                    Equations
                    Instances For

                      The coproduct cocone associated to the explicit finite coproduct.

                      Equations
                      • One or more equations did not get rendered due to their size.
                      Instances For
                        @[simp]
                        theorem CompHaus.finiteCoproduct.isColimit_desc {α : Type w} [Finite α] (X : αCompHausMax) (s : CategoryTheory.Limits.Cocone (CategoryTheory.Discrete.functor X)) :
                        (CompHaus.finiteCoproduct.isColimit X).desc s = CompHaus.finiteCoproduct.desc (fun (a : α) => X a) fun (a : α) => s.app { as := a }

                        The explicit finite coproduct cocone is a colimit cocone.

                        Equations
                        • One or more equations did not get rendered due to their size.
                        Instances For
                          noncomputable def CompHaus.coproductIsoCoproduct {α : Type w} [Finite α] (X : αCompHausMax) :

                          The isomorphism from the explicit finite coproducts to the abstract coproduct.

                          Equations
                          • One or more equations did not get rendered due to their size.
                          Instances For
                            noncomputable def CompHaus.coproductHomeoCoproduct {α : Type w} [Finite α] (X : αCompHausMax) :
                            (CompHaus.finiteCoproduct X).toTop ≃ₜ ( X).toTop

                            The homeomorphism from the explicit finite coproducts to the abstract coproduct.

                            Equations
                            Instances For
                              theorem CompHaus.finiteCoproduct.ι_jointly_surjective {α : Type w} [Finite α] (X : αCompHausMax) (R : (CompHaus.finiteCoproduct X).toTop) :
                              ∃ (a : α) (r : (X a).toTop), R = (CompHaus.finiteCoproduct.ι X a) r
                              theorem CompHaus.finiteCoproduct.ι_desc_apply {α : Type w} [Finite α] (X : αCompHausMax) {B : CompHaus} {π : (a : α) → X a B} (a : α) (x : (CategoryTheory.forget CompHausMax).obj (X a)) :

                              The isomorphism from an arbitrary terminal object of CompHaus to a one-element space.

                              Equations
                              Instances For