diff -r 2606e8c8487d -r 009e176e1010 src/HOL/Topological_Spaces.thy --- a/src/HOL/Topological_Spaces.thy Wed Aug 17 10:26:12 2016 +0200 +++ b/src/HOL/Topological_Spaces.thy Wed Aug 17 16:16:38 2016 +0200 @@ -647,6 +647,16 @@ for x :: "'a::linorder_topology" by (subst at_eq_sup_left_right) (simp add: eventually_sup) +lemma eventually_at_leftI: + assumes "\x. x \ {a<.. P x" "a < b" + shows "eventually P (at_left b)" + using assms unfolding eventually_at_topological by (intro exI[of _ "{a<..}"]) auto + +lemma eventually_at_rightI: + assumes "\x. x \ {a<.. P x" "a < b" + shows "eventually P (at_right a)" + using assms unfolding eventually_at_topological by (intro exI[of _ "{..Tendsto\ @@ -685,6 +695,18 @@ "(LIM x F. f x :> at b within s) \ eventually (\x. f x \ s \ f x \ b) F \ (f \ b) F" by (simp add: at_within_def filterlim_inf filterlim_principal conj_commute) +lemma filterlim_at_withinI: + assumes "filterlim f (nhds c) F" + assumes "eventually (\x. f x \ A - {c}) F" + shows "filterlim f (at c within A) F" + using assms by (simp add: filterlim_at) + +lemma filterlim_atI: + assumes "filterlim f (nhds c) F" + assumes "eventually (\x. f x \ c) F" + shows "filterlim f (at c) F" + using assms by (intro filterlim_at_withinI) simp_all + lemma (in topological_space) topological_tendstoI: "(\S. open S \ l \ S \ eventually (\x. f x \ S) F) \ (f \ l) F" by (auto simp: tendsto_def)