Pullbacks in the category of topological spaces. #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
The explicit pullback cone of X, Y
given by { p : X × Y // f p.1 = g p.2 }
.
Equations
The constructed cone is a limit.
Equations
- Top.pullback_cone_is_limit f g = (Top.pullback_cone f g).is_limit_aux' (λ (s : category_theory.limits.pullback_cone f g), ⟨{to_fun := λ (x : ↥(s.X)), ⟨(⇑(s.fst) x, ⇑(s.snd) x), _⟩, continuous_to_fun := _}, _⟩)
The pullback of two maps can be identified as a subspace of X × Y
.
If the map S ⟶ T
is mono, then there is a description of the image of W ×ₛ X ⟶ Y ×ₜ Z
.
If there is a diagram where the morphisms W ⟶ Y
and X ⟶ Z
are embeddings,
then the induced morphism W ×ₛ X ⟶ Y ×ₜ Z
is also an embedding.
W ⟶ Y ↘ ↘ S ⟶ T ↗ ↗ X ⟶ Z
If there is a diagram where the morphisms W ⟶ Y
and X ⟶ Z
are open embeddings, and S ⟶ T
is mono, then the induced morphism W ×ₛ X ⟶ Y ×ₜ Z
is also an open embedding.
W ⟶ Y
↘ ↘
S ⟶ T
↗ ↗
X ⟶ Z
If X ⟶ S
, Y ⟶ S
are open embeddings, then so is X ×ₛ Y ⟶ S
.