Order connected components of a set #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
In this file we define set.ord_connected_component s x
to be the set of y
such that
set.uIcc x y ⊆ s
and prove some basic facts about this definition. At the moment of writing,
this construction is used only to prove that any linear order with order topology is a T₅ space,
so we only add API needed for this lemma.
Order-connected component of a point x
in a set s
. It is defined as the set of y
such that
set.uIcc x y ⊆ s
. Note that it is empty if and only if x ∉ s
.
Equations
- s.ord_connected_component x = {y : α | set.uIcc x y ⊆ s}
Instances for set.ord_connected_component
Projection from s : set α
to α
sending each order connected component of s
to a single
point of this component.
Equations
- s.ord_connected_proj = λ (x : ↥s), _.some
A set that intersects each order connected component of a set by a single point. Defined as the
range of set.ord_connected_proj s
.
Equations
Given two sets s t : set α
, the set set.order_separating_set s t
is the set of points that
belong both to some set.ord_connected_component tᶜ x
, x ∈ s
, and to some
set.ord_connected_component sᶜ x
, x ∈ t
. In the case of two disjoint closed sets, this is the
union of all open intervals $(a, b)$ such that their endpoints belong to different sets.
Equations
- s.ord_separating_set t = (⋃ (x : α) (H : x ∈ s), tᶜ.ord_connected_component x) ∩ ⋃ (x : α) (H : x ∈ t), sᶜ.ord_connected_component x
An auxiliary neighborhood that will be used in the proof of order_topology.t5_space
.
Equations
- s.ord_t5_nhd t = ⋃ (x : α) (H : x ∈ s), (tᶜ ∩ (s.ord_separating_set t).ord_connected_sectionᶜ).ord_connected_component x