add lemma convergent_Cauchy
authorhuffman
Sun, 24 Sep 2006 04:16:28 +0200
changeset 20691 53cbea20e4d9
parent 20690 136b206327a4
child 20692 6df83a636e67
add lemma convergent_Cauchy
src/HOL/Hyperreal/SEQ.thy
--- a/src/HOL/Hyperreal/SEQ.thy	Sun Sep 24 04:00:46 2006 +0200
+++ b/src/HOL/Hyperreal/SEQ.thy	Sun Sep 24 04:16:28 2006 +0200
@@ -925,6 +925,16 @@
   instantiations for his 'espsilon-delta' proof(s) in this case
   since the NS formulations do not involve existential quantifiers.*}
 
+lemma NSconvergent_NSCauchy: "NSconvergent X \<Longrightarrow> NSCauchy X"
+apply (simp add: NSconvergent_def NSLIMSEQ_def NSCauchy_def, safe)
+apply (auto intro: approx_trans2)
+done
+
+lemma convergent_Cauchy: "convergent X \<Longrightarrow> Cauchy X"
+apply (rule NSconvergent_NSCauchy [THEN NSCauchy_Cauchy])
+apply (simp add: convergent_NSconvergent_iff)
+done
+
 lemma NSCauchy_NSconvergent_iff: "NSCauchy X = NSconvergent (X::nat=>real)"
 apply (simp add: NSconvergent_def NSLIMSEQ_def, safe)
 apply (frule NSCauchy_NSBseq)