src/HOL/Topological_Spaces.thy
changeset 53860 f2d683432580
parent 53859 e6cb01686f7b
child 53946 5431e1392b14
--- a/src/HOL/Topological_Spaces.thy	Tue Sep 24 15:03:49 2013 -0700
+++ b/src/HOL/Topological_Spaces.thy	Tue Sep 24 15:03:49 2013 -0700
@@ -757,6 +757,10 @@
 lemma at_within_empty [simp]: "at a within {} = bot"
   unfolding at_within_def by simp
 
+lemma at_within_union: "at x within (S \<union> T) = sup (at x within S) (at x within T)"
+  unfolding filter_eq_iff eventually_sup eventually_at_filter
+  by (auto elim!: eventually_rev_mp)
+
 lemma at_eq_bot_iff: "at a = bot \<longleftrightarrow> open {a}"
   unfolding trivial_limit_def eventually_at_topological
   by (safe, case_tac "S = {a}", simp, fast, fast)