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

Commit 86c83c3

Browse files
committed
feat(topology): two missing connectedness lemmas (#3626)
From the sphere eversion project.
1 parent ebeeee7 commit 86c83c3

File tree

1 file changed

+12
-0
lines changed

1 file changed

+12
-0
lines changed

src/topology/subset_properties.lean

Lines changed: 12 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -1118,6 +1118,18 @@ lemma subtype.connected_space {s : set α} (h : is_connected s) :
11181118
(subtype.preconnected_space h.is_preconnected).is_preconnected_univ,
11191119
to_nonempty := h.nonempty.to_subtype }
11201120

1121+
lemma is_preconnected_iff_preconnected_space {s : set α} :
1122+
is_preconnected s ↔ preconnected_space s :=
1123+
⟨subtype.preconnected_space,
1124+
begin
1125+
introI,
1126+
simpa using is_preconnected_univ.image (coe : s → α) continuous_subtype_coe.continuous_on
1127+
end
1128+
1129+
lemma is_connected_iff_connected_space {s : set α} : is_connected s ↔ connected_space s :=
1130+
⟨subtype.connected_space,
1131+
λ h, ⟨nonempty_subtype.mp h.2, is_preconnected_iff_preconnected_space.mpr h.1⟩⟩
1132+
11211133
/-- A set `s` is preconnected if and only if
11221134
for every cover by two open sets that are disjoint on `s`,
11231135
it is contained in one of the two covering sets. -/

0 commit comments

Comments
 (0)