Category instance for topological spaces #
We introduce the bundled category TopCat
of topological spaces together with the functors
TopCat.discrete
and TopCat.trivial
from the category of types to TopCat
which equip a type
with the corresponding discrete, resp. trivial, topology. For a proof that these functors are left,
resp. right adjoint to the forgetful functor, see Mathlib.Topology.Category.TopCat.Adjunctions
.
The category of semirings.
- carrier : Type u
The underlying type.
- str : TopologicalSpace ↑self
Instances For
Equations
- TopCat.instCoeSortType = { coe := TopCat.carrier }
The object in TopCat
associated to a type equipped with the appropriate
typeclasses. This is the preferred way to construct a term of TopCat
.
Equations
- TopCat.of X = TopCat.mk✝ X
Instances For
Equations
- One or more equations did not get rendered due to their size.
Typecheck a ContinuousMap
as a morphism in TopCat
.
Equations
Instances For
The results below duplicate the ConcreteCategory
simp lemmas, but we can keep them for dsimp
.
Replace a function coercion for a morphism TopCat.of X ⟶ TopCat.of Y
with the definitionally
equal function coercion for a continuous map C(X, Y)
.
Equations
- TopCat.inhabited = { default := TopCat.of Empty }
The discrete topology on any type.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The trivial topology on any type.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Any homeomorphisms induces an isomorphism in Top
.
Equations
- TopCat.isoOfHomeo f = { hom := TopCat.ofHom ↑f, inv := TopCat.ofHom ↑f.symm, hom_inv_id := ⋯, inv_hom_id := ⋯ }
Instances For
Alias of TopCat.isOpenEmbedding_iff_comp_isIso
.
Alias of TopCat.isOpenEmbedding_iff_comp_isIso'
.
Alias of TopCat.isOpenEmbedding_iff_isIso_comp
.
Alias of TopCat.isOpenEmbedding_iff_isIso_comp'
.