# HG changeset patch # User huffman # Date 1244486899 25200 # Node ID a971fd7d8e45e8f9dc6f62a5c412fc35823348fb # Parent 2ce3583b9261420b15f2e96942319e7be5d8a6f5 generalize lemmas eventually_within_interior, lim_within_interior diff -r 2ce3583b9261 -r a971fd7d8e45 src/HOL/Library/Topology_Euclidean_Space.thy --- a/src/HOL/Library/Topology_Euclidean_Space.thy Mon Jun 08 11:36:35 2009 -0700 +++ b/src/HOL/Library/Topology_Euclidean_Space.thy Mon Jun 08 11:48:19 2009 -0700 @@ -1995,24 +1995,30 @@ text{* For points in the interior, localization of limits makes no difference. *} lemma eventually_within_interior: - fixes x :: "'a::metric_space" assumes "x \ interior S" shows "eventually P (at x within S) \ eventually P (at x)" (is "?lhs = ?rhs") proof- - from assms obtain e where e:"e>0" "\y. dist x y < e \ y \ S" unfolding mem_interior ball_def subset_eq by auto - { assume "?lhs" then obtain d where "d>0" "\xa\S. 0 < dist xa x \ dist xa x < d \ P xa" unfolding eventually_within by auto - hence "?rhs" unfolding eventually_at using e by (auto simp add: dist_commute intro!: add exI[of _ "min e d"]) + from assms obtain T where T: "open T" "x \ T" "T \ S" + unfolding interior_def by fast + { assume "?lhs" + then obtain A where "open A" "x \ A" "\y\A. y \ x \ y \ S \ P y" + unfolding Limits.eventually_within Limits.eventually_at_topological + by auto + with T have "open (A \ T)" "x \ A \ T" "\y\(A \ T). y \ x \ P y" + by auto + then have "?rhs" + unfolding Limits.eventually_at_topological by auto } moreover - { assume "?rhs" hence "?lhs" unfolding eventually_within eventually_at by auto + { assume "?rhs" hence "?lhs" + unfolding Limits.eventually_within + by (auto elim: eventually_elim1) } ultimately - show "?thesis" by auto + show "?thesis" .. qed lemma lim_within_interior: - fixes x :: "'a::metric_space" - fixes l :: "'b::metric_space" (* TODO: generalize *) - shows "x \ interior S ==> ((f ---> l) (at x within S) \ (f ---> l) (at x))" - by (simp add: tendsto_iff eventually_within_interior) + "x \ interior S \ (f ---> l) (at x within S) \ (f ---> l) (at x)" + unfolding tendsto_def by (simp add: eventually_within_interior) lemma netlimit_within_interior: fixes x :: "'a::{perfect_space, real_normed_vector}"