Documentation

Mathlib.Topology.Category.LightProfinite.Limits

Explicit limits and colimits #

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

Main definitions #

The pullback of two morphisms f, g in LightProfinite, 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 isomorphism from the explicit pullback to the abstract pullback.

              Equations
              Instances For
                noncomputable def LightProfinite.pullbackHomeoPullback {X : LightProfinite} {Y : LightProfinite} {B : LightProfinite} (f : X B) (g : Y B) :
                (LightProfinite.pullback f g).toCompHaus.toTop ≃ₜ (CategoryTheory.Limits.pullback f g).toCompHaus.toTop

                The homeomorphism from the explicit pullback to the abstract pullback.

                Equations
                Instances For

                  The "explicit" coproduct of a finite family of objects in LightProfinite, whose underlying profinite set is 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
                      def LightProfinite.finiteCoproduct.desc {α : Type w} [Finite α] (X : αLightProfinite) {B : LightProfinite} (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 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

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

                            Equations
                            Instances For
                              noncomputable def LightProfinite.coproductHomeoCoproduct {α : Type w} [Finite α] (X : αLightProfinite) :
                              (LightProfinite.finiteCoproduct X).toCompHaus.toTop ≃ₜ ( X).toCompHaus.toTop

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

                              Equations
                              Instances For
                                theorem LightProfinite.finiteCoproduct.ι_jointly_surjective {α : Type w} [Finite α] (X : αLightProfinite) (R : (LightProfinite.finiteCoproduct X).toCompHaus.toTop) :
                                ∃ (a : α) (r : (X a).toCompHaus.toTop), R = (LightProfinite.finiteCoproduct.ι X a) r
                                theorem LightProfinite.finiteCoproduct.ι_desc_apply {α : Type w} [Finite α] (X : αLightProfinite) {B : LightProfinite} {π : (a : α) → X a B} (a : α) (x : (CategoryTheory.forget LightProfinite).obj (X a)) :
                                Equations
                                • One or more equations did not get rendered due to their size.
                                Equations
                                • X.instUniqueHomOfPUnit = { default := { toFun := fun (x : X.toCompHaus.toTop) => PUnit.unit, continuous_toFun := }, uniq := }

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

                                Equations
                                Instances For