src/HOL/Topological_Spaces.thy
changeset 63713 009e176e1010
parent 63495 b0f8845e3498
child 63952 354808e9f44b
equal deleted inserted replaced
63712:2606e8c8487d 63713:009e176e1010
   645 lemma eventually_at_split:
   645 lemma eventually_at_split:
   646   "eventually P (at x) \<longleftrightarrow> eventually P (at_left x) \<and> eventually P (at_right x)"
   646   "eventually P (at x) \<longleftrightarrow> eventually P (at_left x) \<and> eventually P (at_right x)"
   647   for x :: "'a::linorder_topology"
   647   for x :: "'a::linorder_topology"
   648   by (subst at_eq_sup_left_right) (simp add: eventually_sup)
   648   by (subst at_eq_sup_left_right) (simp add: eventually_sup)
   649 
   649 
       
   650 lemma eventually_at_leftI:
       
   651   assumes "\<And>x. x \<in> {a<..<b} \<Longrightarrow> P x" "a < b"
       
   652   shows   "eventually P (at_left b)"
       
   653   using assms unfolding eventually_at_topological by (intro exI[of _ "{a<..}"]) auto
       
   654 
       
   655 lemma eventually_at_rightI:
       
   656   assumes "\<And>x. x \<in> {a<..<b} \<Longrightarrow> P x" "a < b"
       
   657   shows   "eventually P (at_right a)"
       
   658   using assms unfolding eventually_at_topological by (intro exI[of _ "{..<b}"]) auto
       
   659 
   650 
   660 
   651 subsubsection \<open>Tendsto\<close>
   661 subsubsection \<open>Tendsto\<close>
   652 
   662 
   653 abbreviation (in topological_space)
   663 abbreviation (in topological_space)
   654   tendsto :: "('b \<Rightarrow> 'a) \<Rightarrow> 'a \<Rightarrow> 'b filter \<Rightarrow> bool"  (infixr "\<longlongrightarrow>" 55)
   664   tendsto :: "('b \<Rightarrow> 'a) \<Rightarrow> 'a \<Rightarrow> 'b filter \<Rightarrow> bool"  (infixr "\<longlongrightarrow>" 55)
   682   by (blast intro: tendsto_mono at_le)
   692   by (blast intro: tendsto_mono at_le)
   683 
   693 
   684 lemma filterlim_at:
   694 lemma filterlim_at:
   685   "(LIM x F. f x :> at b within s) \<longleftrightarrow> eventually (\<lambda>x. f x \<in> s \<and> f x \<noteq> b) F \<and> (f \<longlongrightarrow> b) F"
   695   "(LIM x F. f x :> at b within s) \<longleftrightarrow> eventually (\<lambda>x. f x \<in> s \<and> f x \<noteq> b) F \<and> (f \<longlongrightarrow> b) F"
   686   by (simp add: at_within_def filterlim_inf filterlim_principal conj_commute)
   696   by (simp add: at_within_def filterlim_inf filterlim_principal conj_commute)
       
   697 
       
   698 lemma filterlim_at_withinI:
       
   699   assumes "filterlim f (nhds c) F"
       
   700   assumes "eventually (\<lambda>x. f x \<in> A - {c}) F"
       
   701   shows   "filterlim f (at c within A) F"
       
   702   using assms by (simp add: filterlim_at) 
       
   703 
       
   704 lemma filterlim_atI:
       
   705   assumes "filterlim f (nhds c) F"
       
   706   assumes "eventually (\<lambda>x. f x \<noteq> c) F"
       
   707   shows   "filterlim f (at c) F"
       
   708   using assms by (intro filterlim_at_withinI) simp_all
   687 
   709 
   688 lemma (in topological_space) topological_tendstoI:
   710 lemma (in topological_space) topological_tendstoI:
   689   "(\<And>S. open S \<Longrightarrow> l \<in> S \<Longrightarrow> eventually (\<lambda>x. f x \<in> S) F) \<Longrightarrow> (f \<longlongrightarrow> l) F"
   711   "(\<And>S. open S \<Longrightarrow> l \<in> S \<Longrightarrow> eventually (\<lambda>x. f x \<in> S) F) \<Longrightarrow> (f \<longlongrightarrow> l) F"
   690   by (auto simp: tendsto_def)
   712   by (auto simp: tendsto_def)
   691 
   713