Skip to content

Commit

Permalink
feat(topology/algebra/order/intermediate_value): intervals are connec…
Browse files Browse the repository at this point in the history
…ted (#16473)

`topology.algebra.order.intermediate_value` has a series of lemmas that different kinds of intervals are preconnected.  Add a corresponding series of lemmas that intervals are connected (with appropriate extra conditions on the order or the endpoints as needed).
  • Loading branch information
jsm28 committed Sep 13, 2022
1 parent 4ff1021 commit c64fb26
Showing 1 changed file with 22 additions and 0 deletions.
22 changes: 22 additions & 0 deletions src/topology/algebra/order/intermediate_value.lean
Expand Up @@ -426,6 +426,28 @@ lemma is_preconnected_Ioo : is_preconnected (Ioo a b) := ord_connected_Ioo.is_pr
lemma is_preconnected_Ioc : is_preconnected (Ioc a b) := ord_connected_Ioc.is_preconnected
lemma is_preconnected_Ico : is_preconnected (Ico a b) := ord_connected_Ico.is_preconnected

lemma is_connected_Ici : is_connected (Ici a) := ⟨nonempty_Ici, is_preconnected_Ici⟩

lemma is_connected_Iic : is_connected (Iic a) := ⟨nonempty_Iic, is_preconnected_Iic⟩

lemma is_connected_Ioi [no_max_order α] : is_connected (Ioi a) :=
⟨nonempty_Ioi, is_preconnected_Ioi⟩

lemma is_connected_Iio [no_min_order α] : is_connected (Iio a) :=
⟨nonempty_Iio, is_preconnected_Iio⟩

lemma is_connected_Icc (h : a ≤ b) : is_connected (Icc a b) :=
⟨nonempty_Icc.2 h, is_preconnected_Icc⟩

lemma is_connected_Ioo (h : a < b) : is_connected (Ioo a b) :=
⟨nonempty_Ioo.2 h, is_preconnected_Ioo⟩

lemma is_connected_Ioc (h : a < b) : is_connected (Ioc a b) :=
⟨nonempty_Ioc.2 h, is_preconnected_Ioc⟩

lemma is_connected_Ico (h : a < b) : is_connected (Ico a b) :=
⟨nonempty_Ico.2 h, is_preconnected_Ico⟩

@[priority 100]
instance ordered_connected_space : preconnected_space α :=
⟨ord_connected_univ.is_preconnected⟩
Expand Down

0 comments on commit c64fb26

Please sign in to comment.