src/HOL/Hyperreal/Lim.thy
changeset 23441 ee218296d635
parent 23127 56ee8105c002
child 27435 b3f8e9bdf9a7
--- a/src/HOL/Hyperreal/Lim.thy	Wed Jun 20 17:34:44 2007 +0200
+++ b/src/HOL/Hyperreal/Lim.thy	Wed Jun 20 19:49:14 2007 +0200
@@ -619,7 +619,7 @@
       fix e::real
       assume "0 < e"
         (* choose no such that inverse (real (Suc n)) < e *)
-      have "\<exists>no. inverse (real (Suc no)) < e" by (rule reals_Archimedean)
+      then have "\<exists>no. inverse (real (Suc no)) < e" by (rule reals_Archimedean)
       then obtain m where nodef: "inverse (real (Suc m)) < e" by auto
       show "\<exists>no. \<forall>n. no \<le> n --> \<bar>?F n - a\<bar> < e"
       proof (intro exI allI impI)
@@ -628,7 +628,7 @@
         have "\<bar>?F n - a\<bar> < inverse (real (Suc n))"
           by (rule F2)
         also have "inverse (real (Suc n)) \<le> inverse (real (Suc m))"
-          by auto
+          using mlen by auto
         also from nodef have
           "inverse (real (Suc m)) < e" .
         finally show "\<bar>?F n - a\<bar> < e" .
@@ -664,10 +664,10 @@
    (X -- a --> L)"
 proof
   assume "\<forall>S. (\<forall>n. S n \<noteq> a) \<and> S ----> a \<longrightarrow> (\<lambda>n. X (S n)) ----> L"
-  show "X -- a --> L" by (rule LIMSEQ_SEQ_conv2)
+  thus "X -- a --> L" by (rule LIMSEQ_SEQ_conv2)
 next
   assume "(X -- a --> L)"
-  show "\<forall>S. (\<forall>n. S n \<noteq> a) \<and> S ----> a \<longrightarrow> (\<lambda>n. X (S n)) ----> L" by (rule LIMSEQ_SEQ_conv1)
+  thus "\<forall>S. (\<forall>n. S n \<noteq> a) \<and> S ----> a \<longrightarrow> (\<lambda>n. X (S n)) ----> L" by (rule LIMSEQ_SEQ_conv1)
 qed
 
 end