Documentation

Mathlib.Topology.Category.TopCat.Limits.Basic

The category of topological spaces has all limits and colimits #

Further, these limits and colimits are preserved by the forgetful functor --- that is, the underlying types are just the limits in the category of types.

@[inline, reducible]
abbrev TopCatMax :
Type ((max u v) + 1)

Universe inequalities in Mathlib 3 are expressed through use of max u v. Unfortunately, this leads to unbound universes which cannot be solved for during unification, eg max u v =?= max v ?. The current solution is to wrap Type max u v in TypeMax.{u,v} to expose both universe parameters directly.

Similarly, for other concrete categories for which we need to refer to the maximum of two universes (e.g. any category for which we are constructing limits), we need an analogous abbreviation.

Equations
Instances For

    A choice of limit cone for a functor F : J ⥤ TopCat. Generally you should just use limit.cone F, unless you need the actual definition (which is in terms of Types.limitCone).

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

      A choice of limit cone for a functor F : J ⥤ TopCat whose topology is defined as an infimum of topologies infimum. Generally you should just use limit.cone F, unless you need the actual definition (which is in terms of Types.limitCone).

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

        The chosen cone TopCat.limitCone F for a functor F : J ⥤ TopCat is a limit cone. Generally you should just use limit.isLimit F, unless you need the actual definition (which is in terms of Types.limitConeIsLimit).

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

          The chosen cone TopCat.limitConeInfi F for a functor F : J ⥤ TopCat is a limit cone. Generally you should just use limit.isLimit F, unless you need the actual definition (which is in terms of Types.limitConeIsLimit).

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

            A choice of colimit cocone for a functor F : J ⥤ TopCat. Generally you should just use colimit.cocone F, unless you need the actual definition (which is in terms of Types.colimitCocone).

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

              The chosen cocone TopCat.colimitCocone F for a functor F : J ⥤ TopCat is a colimit cocone. Generally you should just use colimit.isColimit F, unless you need the actual definition (which is in terms of Types.colimitCoconeIsColimit).

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