src/HOL/Topological_Spaces.thy
changeset 68802 3974935e0252
parent 68721 53ad5c01be3f
child 68860 f443ec10447d
equal deleted inserted replaced
68801:c898c2b1fd58 68802:3974935e0252
   454 
   454 
   455 
   455 
   456 subsubsection \<open>Topological filters\<close>
   456 subsubsection \<open>Topological filters\<close>
   457 
   457 
   458 definition (in topological_space) nhds :: "'a \<Rightarrow> 'a filter"
   458 definition (in topological_space) nhds :: "'a \<Rightarrow> 'a filter"
   459   where "nhds a = (INF S:{S. open S \<and> a \<in> S}. principal S)"
   459   where "nhds a = (INF S\<in>{S. open S \<and> a \<in> S}. principal S)"
   460 
   460 
   461 definition (in topological_space) at_within :: "'a \<Rightarrow> 'a set \<Rightarrow> 'a filter"
   461 definition (in topological_space) at_within :: "'a \<Rightarrow> 'a set \<Rightarrow> 'a filter"
   462     ("at (_)/ within (_)" [1000, 60] 60)
   462     ("at (_)/ within (_)" [1000, 60] 60)
   463   where "at a within s = inf (nhds a) (principal (s - {a}))"
   463   where "at a within s = inf (nhds a) (principal (s - {a}))"
   464 
   464 
   470 
   470 
   471 abbreviation (in order_topology) at_left :: "'a \<Rightarrow> 'a filter"
   471 abbreviation (in order_topology) at_left :: "'a \<Rightarrow> 'a filter"
   472   where "at_left x \<equiv> at x within {..< x}"
   472   where "at_left x \<equiv> at x within {..< x}"
   473 
   473 
   474 lemma (in topological_space) nhds_generated_topology:
   474 lemma (in topological_space) nhds_generated_topology:
   475   "open = generate_topology T \<Longrightarrow> nhds x = (INF S:{S\<in>T. x \<in> S}. principal S)"
   475   "open = generate_topology T \<Longrightarrow> nhds x = (INF S\<in>{S\<in>T. x \<in> S}. principal S)"
   476   unfolding nhds_def
   476   unfolding nhds_def
   477 proof (safe intro!: antisym INF_greatest)
   477 proof (safe intro!: antisym INF_greatest)
   478   fix S
   478   fix S
   479   assume "generate_topology T S" "x \<in> S"
   479   assume "generate_topology T S" "x \<in> S"
   480   then show "(INF S:{S \<in> T. x \<in> S}. principal S) \<le> principal S"
   480   then show "(INF S\<in>{S \<in> T. x \<in> S}. principal S) \<le> principal S"
   481     by induct
   481     by induct
   482       (auto intro: INF_lower order_trans simp: inf_principal[symmetric] simp del: inf_principal)
   482       (auto intro: INF_lower order_trans simp: inf_principal[symmetric] simp del: inf_principal)
   483 qed (auto intro!: INF_lower intro: generate_topology.intros)
   483 qed (auto intro!: INF_lower intro: generate_topology.intros)
   484 
   484 
   485 lemma (in topological_space) eventually_nhds:
   485 lemma (in topological_space) eventually_nhds: