Underlying topological space of fibre product of schemes #
Let f : X ⟶ S
and g : Y ⟶ S
be morphisms of schemes. In this file we describe the underlying
topological space of pullback f g
, i.e. the fiber product X ×[S] Y
.
Main results #
AlgebraicGeometry.Scheme.Pullback.carrierEquiv
: The bijective correspondence between the points ofX ×[S] Y
and pairs(z, p)
of triplesz = (x, y, s)
withf x = s = g y
and prime idealsq
ofκ(x) ⊗[κ(s)] κ(y)
.AlgebraicGeometry.Scheme.Pullback.exists_preimage
: For every triple(x, y, s)
withf x = s = g y
, there existsz : X ×[S] Y
lying abovex
andy
.
We also give the ranges of pullback.fst
, pullback.snd
and pullback.map
.
A Triplet
over f : X ⟶ S
and g : Y ⟶ S
is a triple of points x : X
, y : Y
,
s : S
such that f x = s = f y
.
- x : ↑↑X.toPresheafedSpace
The point of
X
. - y : ↑↑Y.toPresheafedSpace
The point of
Y
. - s : ↑↑S.toPresheafedSpace
- hx : f.base self.x = self.s
- hy : g.base self.y = self.s
Instances For
Make a triplet from x : X
and y : Y
such that f x = g y
.
Equations
- AlgebraicGeometry.Scheme.Pullback.Triplet.mk' x y h = { x := x, y := y, s := g.base y, hx := h, hy := ⋯ }
Instances For
Given x : X
and y : Y
such that f x = s = g y
, this is κ(x) ⊗[κ(s)] κ(y)
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- ⋯ = ⋯
Given x : X
and y : Y
such that f x = s = g y
, this is the
canonical map κ(x) ⟶ κ(x) ⊗[κ(s)] κ(y)
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Given x : X
and y : Y
such that f x = s = g y
, this is the
canonical map κ(y) ⟶ κ(x) ⊗[κ(s)] κ(y)
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Given propositionally equal triplets T₁
and T₂
over f
and g
, the corresponding
T₁.tensor
and T₂.tensor
are isomorphic.
Instances For
Given x : X
, y : Y
and s : S
such that f x = s = g y
,
this is Spec (κ(x) ⊗[κ(s)] κ(y)) ⟶ X ×ₛ Y
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Given t : X ×[S] Y
, it maps to X
and Y
with same image in S
, yielding a
Triplet f g
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Given t : X ×[S] Y
with projections to X
, Y
and S
denoted by x
, y
and s
respectively, this is the canonical map κ(x) ⊗[κ(s)] κ(y) ⟶ κ(t)
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
If t
is a point in X ×[S] Y
above (x, y, s)
, then this is the image of the unique
point of Spec κ(s)
in Spec κ(x) ⊗[κ(s)] κ(y)
.
Equations
Instances For
A helper lemma to work with AlgebraicGeometry.Scheme.Pullback.carrierEquiv
.
The points of the underlying topological space of X ×[S] Y
bijectively correspond to
pairs of triples x : X
, y : Y
, s : S
with f x = s = f y
and prime ideals of
κ(x) ⊗[κ(s)] κ(y)
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Given a triple (x, y, s)
with f x = s = f y
there exists t : X ×[S] Y
above
x
and ỳ
. For the unpacked version without Triplet
, see
AlgebraicGeometry.Scheme.Pullback.exists_preimage
.
If f : X ⟶ S
and g : Y ⟶ S
are morphisms of schemes and x : X
and y : Y
are points such
that f x = g y
, then there exists z : X ×[S] Y
lying above x
and y
.
In other words, the map from the underlying topological space of X ×[S] Y
to the fiber product
of the underlying topological spaces of X
and Y
over S
is surjective.