@@ -74,21 +74,8 @@ show A = sequential_closure A, from subset.antisymm
74
74
/-- The sequential closure of a set is contained in the closure of that set.
75
75
The converse is not true. -/
76
76
lemma sequential_closure_subset_closure (M : set α) : sequential_closure M ⊆ closure M :=
77
- show ∀ p, p ∈ sequential_closure M → p ∈ closure M, from
78
- assume p,
79
- assume : ∃ x : ℕ → α, (∀ n : ℕ, ((x n) ∈ M)) ∧ (x ⟶ p),
80
- let ⟨x, ⟨_, _⟩⟩ := this in
81
- show p ∈ closure M, from
82
- -- we have to show that p is in the closure of M
83
- -- using mem_closure_iff, this is equivalent to proving that every open neighbourhood
84
- -- has nonempty intersection with M, but this is witnessed by our sequence x
85
- suffices ∀ O, is_open O → p ∈ O → O ∩ M ≠ ∅, from mem_closure_iff.mpr this ,
86
- have ∀ (U : set α), p ∈ U → is_open U → (∃ n0, ∀ n, n ≥ n0 → x n ∈ U), by rwa[←topological_space.seq_tendsto_iff],
87
- assume O is_open_O p_in_O,
88
- let ⟨n0, _⟩ := this O ‹p ∈ O› ‹is_open O› in
89
- have (x n0) ∈ O, from ‹∀ n ≥ n0, x n ∈ O› n0 (show n0 ≥ n0, from le_refl n0),
90
- have (x n0) ∈ O ∩ M, from ⟨this , ‹∀n, x n ∈ M› n0⟩,
91
- set.ne_empty_of_mem this
77
+ assume p ⟨x, xM, xp⟩,
78
+ mem_closure_of_tendsto at_top_ne_bot xp (univ_mem_sets' xM)
92
79
93
80
/-- A set is sequentially closed if it is closed. -/
94
81
lemma is_seq_closed_of_is_closed (M : set α) (_ : is_closed M) : is_seq_closed M :=
0 commit comments