The adjunction between light condensed sets and topological spaces #
This file defines the functor lightCondSetToTopCat : LightCondSet.{u} ⥤ TopCat.{u}
which is
left adjoint to topCatToLightCondSet : TopCat.{u} ⥤ LightCondSet.{u}
. We prove that the counit
is bijective (but not in general an isomorphism) and conclude that the right adjoint is faithful.
The counit is an isomorphism for sequential spaces, and we conclude that the functor
topCatToLightCondSet
is fully faithful when restricted to sequential spaces.
Let X
be a light condensed set. We define a topology on X(*)
as the quotient topology of
all the maps from light profinite sets S
to X(*)
, corresponding to elements of X(S)
.
In other words, the topology coinduced by the map LightCondSet.coinducingCoprod
above.
Equations
- X.underlyingTopologicalSpace = TopologicalSpace.coinduced (LightCondSet.coinducingCoprod X) inferInstance
Instances For
The object part of the functor LightCondSet ⥤ TopCat
Equations
- X.toTopCat = TopCat.of (X.val.obj (Opposite.op (LightProfinite.of PUnit.{?u.11 + 1} )))
Instances For
The map part of the functor LightCondSet ⥤ TopCat
Equations
- LightCondSet.toTopCatMap f = { toFun := f.val.app (Opposite.op (LightProfinite.of PUnit.{?u.31 + 1} )), continuous_toFun := ⋯ }
Instances For
The functor LightCondSet ⥤ TopCat
Equations
- One or more equations did not get rendered due to their size.
Instances For
The counit of the adjunction lightCondSetToTopCat ⊣ topCatToLightCondSet
Equations
- LightCondSet.topCatAdjunctionCounit X = { toFun := fun (x : ↑X.toLightCondSet.toTopCat) => x.toFun PUnit.unit, continuous_toFun := ⋯ }
Instances For
The counit of the adjunction lightCondSetToTopCat ⊣ topCatToLightCondSet
is always bijective,
but not an isomorphism in general (the inverse isn't continuous unless X
is sequential).
Equations
- One or more equations did not get rendered due to their size.
Instances For
The unit of the adjunction lightCondSetToTopCat ⊣ topCatToLightCondSet
Equations
- One or more equations did not get rendered due to their size.
Instances For
The adjunction lightCondSetToTopCat ⊣ topCatToLightCondSet
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- ⋯ = ⋯
Equations
- ⋯ = ⋯
Equations
- ⋯ = ⋯
The functor from light condensed sets to topological spaces lands in sequential spaces.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The functor from topological spaces to light condensed sets restricted to sequential spaces.
Equations
Instances For
The adjunction lightCondSetToTopCat ⊣ topCatToLightCondSet
restricted to sequential
spaces.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The counit of the adjunction lightCondSetToSequential ⊣ sequentialToLightCondSet
is a homeomorphism.
Note: for now, we only have ℕ∪{∞}
as a light profinite set at universe level 0, which is why we
can only prove this for X : TopCat.{0}
.
Equations
- LightCondSet.sequentialAdjunctionHomeo X = { toEquiv := LightCondSet.topCatAdjunctionCounitEquiv X, continuous_toFun := ⋯, continuous_invFun := ⋯ }
Instances For
The counit of the adjunction lightCondSetToSequential ⊣ sequentialToLightCondSet
is an isomorphism.
Note: for now, we only have ℕ∪{∞}
as a light profinite set at universe level 0, which is why we
can only prove this for X : Sequential.{0}
.
Equations
Instances For
The functor from topological spaces to light condensed sets restricted to sequential spaces is fully faithful.
Note: for now, we only have ℕ∪{∞}
as a light profinite set at universe level 0, which is why we
can only prove this for the functor Sequential.{0} ⥤ LightCondSet.{0}
.
Equations
- LightCondSet.fullyFaithfulSequentialToLightCondSet = LightCondSet.sequentialAdjunction.fullyFaithfulROfIsIsoCounit