diff -r 8f3625167c76 -r 93943da0a010 src/HOL/Multivariate_Analysis/Cartesian_Euclidean_Space.thy --- a/src/HOL/Multivariate_Analysis/Cartesian_Euclidean_Space.thy Mon Sep 12 11:39:29 2011 -0700 +++ b/src/HOL/Multivariate_Analysis/Cartesian_Euclidean_Space.thy Mon Sep 12 11:54:20 2011 -0700 @@ -1817,7 +1817,7 @@ apply(induct_tac n) apply simp using assms(2) apply(erule_tac x="na" in allE) by(auto simp add: not_less_eq_eq) } hence "\m n. m \ n \ dest_vec1 (s m) \ dest_vec1 (s n)" by auto then obtain l where "\e>0. \N. \n\N. \dest_vec1 (s n) - l\ < e" using convergent_bounded_monotone[OF a] unfolding monoseq_def by auto - thus ?thesis unfolding Lim_sequentially apply(rule_tac x="vec1 l" in exI) + thus ?thesis unfolding LIMSEQ_def apply(rule_tac x="vec1 l" in exI) unfolding dist_norm unfolding abs_dest_vec1 by auto qed