Skip to content

Commit

Permalink
feat(topological_structures): frontier_lt_subset_eq
Browse files Browse the repository at this point in the history
Based on a suggestion by Luca Gerolla
  • Loading branch information
digama0 committed Aug 16, 2018
1 parent d468921 commit 032e21d
Show file tree
Hide file tree
Showing 2 changed files with 8 additions and 1 deletion.
5 changes: 4 additions & 1 deletion analysis/topology/topological_space.lean
Original file line number Diff line number Diff line change
Expand Up @@ -277,6 +277,9 @@ lemma frontier_eq_closure_inter_closure {s : set α} :
frontier s = closure s ∩ closure (- s) :=
by rw [closure_compl, frontier, diff_eq]

@[simp] lemma frontier_compl (s : set α) : frontier (-s) = frontier s :=
by simp [frontier_eq_closure_inter_closure, inter_comm]

/-- neighbourhood filter -/
def nhds (a : α) : filter α := (⨅ s ∈ {s : set α | a ∈ s ∧ is_open s}, principal s)

Expand Down Expand Up @@ -1162,7 +1165,7 @@ begin
let B' := {b ∈ B | ∃ s ∈ S, b ⊆ s},
rcases axiom_of_choice (λ b:B', b.2.2) with ⟨f, hf⟩,
change B' → set α at f,
haveI : encodable B' := (countable_subset (sep_subset _ _) cB).to_encodable,
haveI : encodable B' := (countable_subset (sep_subset _ _) cB).to_encodable,
have : range f ⊆ S := range_subset_iff.2 (λ x, (hf x).fst),
exact ⟨_, countable_range f, this,
subset.antisymm (sUnion_subset_sUnion this) $
Expand Down
4 changes: 4 additions & 0 deletions analysis/topology/topological_structures.lean
Original file line number Diff line number Diff line change
Expand Up @@ -344,6 +344,10 @@ le_antisymm
have b ∈ interior {b | f b ≤ g b}, from this hb,
by exact hb₂ this)

lemma frontier_lt_subset_eq : frontier {b | f b < g b} ⊆ {b | f b = g b} :=
by rw ← frontier_compl;
convert frontier_le_subset_eq hg hf; simp [ext_iff, eq_comm]

lemma continuous_max : continuous (λb, max (f b) (g b)) :=
have ∀b∈frontier {b | f b ≤ g b}, g b = f b, from assume b hb, (frontier_le_subset_eq hf hg hb).symm,
continuous_if this hg hf
Expand Down

0 comments on commit 032e21d

Please sign in to comment.