Documentation

Mathlib.Topology.Category.CompHausLike.Limits

Explicit limits and colimits #

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

So far, we have the following:

@[reducible, inline]
abbrev CompHausLike.HasExplicitFiniteCoproduct {P : TopCatProp} {α : Type w} (X : αCompHausLike P) :

A typeclass describing the property that forming the disjoint union is stable under the property P.

Equations
Instances For

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

    Equations
    Instances For

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

      Equations
      Instances For

        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
          @[reducible, inline]

          The coproduct cocone associated to the explicit finite coproduct.

          Equations
          Instances For

            The explicit finite coproduct cocone is a colimit cocone.

            Equations
            • One or more equations did not get rendered due to their size.
            Instances For
              theorem CompHausLike.finiteCoproduct.ι_jointly_surjective {P : TopCatProp} {α : Type w} [Finite α] (X : αCompHausLike P) [CompHausLike.HasExplicitFiniteCoproduct X] (R : (CompHausLike.finiteCoproduct X).toTop) :
              ∃ (a : α) (r : (X a).toTop), R = (CompHausLike.finiteCoproduct.ι X a) r
              theorem CompHausLike.finiteCoproduct.ι_desc_apply {P : TopCatProp} {α : Type w} [Finite α] (X : αCompHausLike P) [CompHausLike.HasExplicitFiniteCoproduct X] {B : CompHausLike P} {π : (a : α) → X a B} (a : α) (x : (CategoryTheory.forget (CompHausLike P)).obj (X a)) :

              A typeclass describing the property that forming all finite disjoint unions is stable under the property P.

              Instances

                The inclusion maps into the explicit finite coproduct are open embeddings.

                The inclusion maps into the abstract finite coproduct are open embeddings.

                The functor to TopCat preserves finite coproducts if they exist.

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

                The functor to another CompHausLike preserves finite coproducts if they exist.

                Equations
                • One or more equations did not get rendered due to their size.
                @[reducible, inline]
                abbrev CompHausLike.HasExplicitPullback {P : TopCatProp} {X : CompHausLike P} {Y : CompHausLike P} {B : CompHausLike P} (f : X B) (g : Y B) :

                A typeclass describing the property that an explicit pullback is stable under the property P.

                Equations
                Instances For

                  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

                    The projection from the pullback to the first component.

                    Equations
                    Instances For

                      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
                        Instances For

                          The pullback cone whose cone point is the explicit pullback.

                          Equations
                          Instances For

                            The explicit pullback cone is a limit cone.

                            Equations
                            Instances For

                              The functor to TopCat creates pullbacks if they exist.

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

                              The functor to TopCat preserves pullbacks.

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

                              The functor to another CompHausLike preserves pullbacks.

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

                              A typeclass describing the property that forming all explicit pullbacks is stable under the property P.

                              Instances

                                A typeclass describing the property that explicit pullbacks along inclusion maps into disjoint unions is stable under the property P.

                                Instances

                                  The functor to TopCat preserves pullbacks of inclusions if they exist.

                                  Equations
                                  • CompHausLike.instPreservesPullbacksOfInclusionsTopCatCompHausLikeToTopOfHasExplicitPullbacksOfInclusions = CategoryTheory.PreservesPullbacksOfInclusions.mk