diff -r 1cc4ab4b7ff7 -r 0a5b7b818d65 src/HOL/Library/Product_Vector.thy --- a/src/HOL/Library/Product_Vector.thy Tue May 04 10:06:05 2010 -0700 +++ b/src/HOL/Library/Product_Vector.thy Tue May 04 10:42:47 2010 -0700 @@ -312,18 +312,6 @@ (simp add: subsetD [OF `A \ B \ S`]) qed -lemma LIM_fst: "f -- x --> a \ (\x. fst (f x)) -- x --> fst a" -unfolding LIM_conv_tendsto by (rule tendsto_fst) - -lemma LIM_snd: "f -- x --> a \ (\x. snd (f x)) -- x --> snd a" -unfolding LIM_conv_tendsto by (rule tendsto_snd) - -lemma LIM_Pair: - assumes "f -- x --> a" and "g -- x --> b" - shows "(\x. (f x, g x)) -- x --> (a, b)" -using assms unfolding LIM_conv_tendsto -by (rule tendsto_Pair) - lemma Cauchy_fst: "Cauchy X \ Cauchy (\n. fst (X n))" unfolding Cauchy_def by (fast elim: le_less_trans [OF dist_fst_le]) @@ -348,7 +336,7 @@ lemma isCont_Pair [simp]: "\isCont f x; isCont g x\ \ isCont (\x. (f x, g x)) x" - unfolding isCont_def by (rule LIM_Pair) + unfolding isCont_def by (rule tendsto_Pair) subsection {* Product is a complete metric space *}