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.
Main definitions #
HasExplicitFiniteCoproducts
: A typeclass describing the property that forming all finite disjoint unions is stable under the propertyP
.- Given this property, we deduce that
CompHausLike P
has finite coproducts and the inclusion functors to otherCompHausLike P'
and toTopCat
preserve them.
- Given this property, we deduce that
HasExplicitPullbacks
: A typeclass describing the property that forming all "explicit pullbacks" is stable under the propertyP
. Here, explicit pullbacks are defined as a subset of the product.- Given this property, we deduce that
CompHausLike P
has pullbacks and the inclusion functors to otherCompHausLike P'
and toTopCat
preserve them. - We also define a variant
HasExplicitPullbacksOfInclusions
which is says that explicit pullbacks along inclusion maps into finite disjoint unions exist.Stonean
has this property but not the stronger one.
- Given this property, we deduce that
Main results #
- Given
[HasExplicitPullbacksOfInclusions P]
(which is implied by[HasExplicitPullbacks P]
), we provide an instanceFinitaryExtensive (CompHausLike P)
.
A typeclass describing the property that forming the disjoint union is stable under the
property P
.
Equations
- CompHausLike.HasExplicitFiniteCoproduct X = CompHausLike.HasProp P ((a : α) × ↑(X a).toTop)
Instances For
The coproduct of a finite family of objects in CompHaus
, constructed as the disjoint
union with its usual topology.
Equations
- CompHausLike.finiteCoproduct X = CompHausLike.of P ((a : α) × ↑(X a).toTop)
Instances For
The inclusion of one of the factors into the explicit finite coproduct.
Equations
- CompHausLike.finiteCoproduct.ι X a = { toFun := fun (x : ↑(X a).toTop) => ⟨a, x⟩, continuous_toFun := ⋯ }
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
- CompHausLike.finiteCoproduct.desc X e = { toFun := fun (x : ↑(CompHausLike.finiteCoproduct X).toTop) => match x with | ⟨a, x⟩ => (e a) x, continuous_toFun := ⋯ }
Instances For
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
A typeclass describing the property that forming all finite disjoint unions is stable under the
property P
.
- hasProp {α : Type w} [Finite α] (X : α → CompHausLike P) : CompHausLike.HasExplicitFiniteCoproduct X
Instances
The inclusion maps into the explicit finite coproduct are open embeddings.
Alias of CompHausLike.finiteCoproduct.isOpenEmbedding_ι
.
The inclusion maps into the explicit finite coproduct are open embeddings.
The inclusion maps into the abstract finite coproduct are open embeddings.
Alias of CompHausLike.Sigma.isOpenEmbedding_ι
.
The inclusion maps into the abstract finite coproduct are open embeddings.
The functor to TopCat
preserves finite coproducts if they exist.
The functor to another CompHausLike
preserves finite coproducts if they exist.
A typeclass describing the property that an explicit pullback is stable under the property P
.
Equations
- CompHausLike.HasExplicitPullback f g = CompHausLike.HasProp P ↑{xy : ↑X.toTop × ↑Y.toTop | f xy.1 = g xy.2}
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
- CompHausLike.pullback f g = CompHausLike.of P ↑{xy : ↑X.toTop × ↑Y.toTop | f xy.1 = g xy.2}
Instances For
The projection from the pullback to the first component.
Equations
- CompHausLike.pullback.fst f g = { toFun := fun (x : ↑(CompHausLike.pullback f g).toTop) => match x with | ⟨(x, snd), property⟩ => x, continuous_toFun := ⋯ }
Instances For
The projection from the pullback to the second component.
Equations
- CompHausLike.pullback.snd f g = { toFun := fun (x : ↑(CompHausLike.pullback f g).toTop) => match x with | ⟨(fst, y), property⟩ => y, continuous_toFun := ⋯ }
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
- CompHausLike.pullback.lift f g a b w = { toFun := fun (z : ↑Z.toTop) => ⟨(a z, b z), ⋯⟩, continuous_toFun := ⋯ }
Instances For
The pullback cone whose cone point is the explicit pullback.
Equations
Instances For
The explicit pullback cone is a limit cone.
Equations
- CompHausLike.pullback.isLimit f g = (CompHausLike.pullback.cone f g).isLimitAux (fun (s : CategoryTheory.Limits.PullbackCone f g) => CompHausLike.pullback.lift f g s.fst s.snd ⋯) ⋯ ⋯ ⋯
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.
The functor to another CompHausLike
preserves pullbacks.
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
.
- hasProp {X Y Z : CompHausLike P} (f : Z ⟶ X ⨿ Y) : CompHausLike.HasExplicitPullback CategoryTheory.Limits.coprod.inl f
Instances
The functor to TopCat
preserves pullbacks of inclusions if they exist.
A one-element space is terminal in CompHaus
Equations
- CompHausLike.isTerminalPUnit = CategoryTheory.Limits.IsTerminal.ofUnique (CompHausLike.of P PUnit.{?u.30 + 1})