Lifting topological spaces to a higher universe #
In this file, we construct the functor uliftFunctor.{v, u} : TopCat.{u} ⥤ TopCat.{max u v}
which sends a topological space X : Type u
to a homeomorphic space in Type (max u v)
.
The functor which sends a topological space in Type u
to a homeomorphic
space in Type (max u v)
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Given X : TopCat.{u}
, this is the homeomorphism X ≃ₜ uliftFunctor.{v}.obj X
.
Equations
Instances For
@[simp]
@[simp]
theorem
TopCat.uliftFunctorObjHomeo_symm_naturality_apply
{X Y : TopCat}
(f : X ⟶ Y)
(x : ↑(uliftFunctor.obj X))
:
The ULift
functor on categories of topological spaces is compatible
with the one defined on categories of types.
Equations
Instances For
@[simp]
theorem
TopCat.uliftFunctorCompForgetIso_hom_app
(X : TopCat)
(a✝ : (uliftFunctor.comp (CategoryTheory.forget TopCat)).obj X)
:
@[simp]
theorem
TopCat.uliftFunctorCompForgetIso_inv_app
(X : TopCat)
(a✝ : (uliftFunctor.comp (CategoryTheory.forget TopCat)).obj X)
:
The ULift
functor on categories of topological spaces is fully faithful.
Equations
- One or more equations did not get rendered due to their size.