Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit c64fb26

Browse files
committed
feat(topology/algebra/order/intermediate_value): intervals are connected (#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).
1 parent 4ff1021 commit c64fb26

File tree

1 file changed

+22
-0
lines changed

1 file changed

+22
-0
lines changed

src/topology/algebra/order/intermediate_value.lean

Lines changed: 22 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -426,6 +426,28 @@ lemma is_preconnected_Ioo : is_preconnected (Ioo a b) := ord_connected_Ioo.is_pr
426426
lemma is_preconnected_Ioc : is_preconnected (Ioc a b) := ord_connected_Ioc.is_preconnected
427427
lemma is_preconnected_Ico : is_preconnected (Ico a b) := ord_connected_Ico.is_preconnected
428428

429+
lemma is_connected_Ici : is_connected (Ici a) := ⟨nonempty_Ici, is_preconnected_Ici⟩
430+
431+
lemma is_connected_Iic : is_connected (Iic a) := ⟨nonempty_Iic, is_preconnected_Iic⟩
432+
433+
lemma is_connected_Ioi [no_max_order α] : is_connected (Ioi a) :=
434+
⟨nonempty_Ioi, is_preconnected_Ioi⟩
435+
436+
lemma is_connected_Iio [no_min_order α] : is_connected (Iio a) :=
437+
⟨nonempty_Iio, is_preconnected_Iio⟩
438+
439+
lemma is_connected_Icc (h : a ≤ b) : is_connected (Icc a b) :=
440+
⟨nonempty_Icc.2 h, is_preconnected_Icc⟩
441+
442+
lemma is_connected_Ioo (h : a < b) : is_connected (Ioo a b) :=
443+
⟨nonempty_Ioo.2 h, is_preconnected_Ioo⟩
444+
445+
lemma is_connected_Ioc (h : a < b) : is_connected (Ioc a b) :=
446+
⟨nonempty_Ioc.2 h, is_preconnected_Ioc⟩
447+
448+
lemma is_connected_Ico (h : a < b) : is_connected (Ico a b) :=
449+
⟨nonempty_Ico.2 h, is_preconnected_Ico⟩
450+
429451
@[priority 100]
430452
instance ordered_connected_space : preconnected_space α :=
431453
⟨ord_connected_univ.is_preconnected⟩

0 commit comments

Comments
 (0)