Sober spaces #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
A quasi-sober space is a topological space where every
irreducible closed subset has a generic point.
A sober space is a quasi-sober space where every irreducible closed subset
has a unique generic point. This is if and only if the space is T0, and thus sober spaces can be
stated via [quasi_sober α] [t0_space α]
.
Main definition #
is_generic_point
:x
is the generic point ofS
ifS
is the closure ofx
.quasi_sober
: A space is quasi-sober if every irreducible closed subset has a generic point.
x
is a generic point of S
if S
is the closure of x
.
Equations
- is_generic_point x S = (closure {x} = S)
In a T₀ space, each set has at most one generic point.
- sober : ∀ {S : set α}, is_irreducible S → is_closed S → (∃ (x : α), is_generic_point x S)
A space is sober if every irreducible closed subset has a generic point.
Instances of this typeclass
A generic point of the closure of an irreducible space.
Equations
- hS.generic_point = _.some
A generic point of a sober irreducible space.
Equations
The closed irreducible subsets of a sober space bijects with the points of the space.
Equations
- irreducible_set_equiv_points = {to_equiv := {to_fun := λ (s : ↥{s : set α | is_irreducible s ∧ is_closed s}), _.generic_point, inv_fun := λ (x : α), ⟨closure {x}, _⟩, left_inv := _, right_inv := _}, map_rel_iff' := _}