src/HOL/Hyperreal/SEQ.thy
changeset 15241 a3949068537e
parent 15236 f289e8ba2bb3
child 15251 bb6f072c8d10
equal deleted inserted replaced
15240:e1e6db03beee 15241:a3949068537e
  1094  -- Show we can take subsequential terms arbitrarily far
  1094  -- Show we can take subsequential terms arbitrarily far
  1095     up a sequence
  1095     up a sequence
  1096 Goal "subseq f ==> n \<le> f(n)";
  1096 Goal "subseq f ==> n \<le> f(n)";
  1097 Goal "subseq f ==> \<exists>n. N1 \<le> n & N2 \<le> f(n)";
  1097 Goal "subseq f ==> \<exists>n. N1 \<le> n & N2 \<le> f(n)";
  1098  ---------------------------------------------------------------***)
  1098  ---------------------------------------------------------------***)
       
  1099 
  1099 
  1100 
  1100 ML
  1101 ML
  1101 {*
  1102 {*
  1102 val Cauchy_def = thm"Cauchy_def";
  1103 val Cauchy_def = thm"Cauchy_def";
  1103 val SEQ_Infinitesimal = thm "SEQ_Infinitesimal";
  1104 val SEQ_Infinitesimal = thm "SEQ_Infinitesimal";
  1212 val LIMSEQ_pow = thm "LIMSEQ_pow";
  1213 val LIMSEQ_pow = thm "LIMSEQ_pow";
  1213 val Bseq_realpow = thm "Bseq_realpow";
  1214 val Bseq_realpow = thm "Bseq_realpow";
  1214 val monoseq_realpow = thm "monoseq_realpow";
  1215 val monoseq_realpow = thm "monoseq_realpow";
  1215 val convergent_realpow = thm "convergent_realpow";
  1216 val convergent_realpow = thm "convergent_realpow";
  1216 val NSLIMSEQ_realpow_zero = thm "NSLIMSEQ_realpow_zero";
  1217 val NSLIMSEQ_realpow_zero = thm "NSLIMSEQ_realpow_zero";
  1217 val LIMSEQ_realpow_zero = thm "LIMSEQ_realpow_zero";
       
  1218 val LIMSEQ_divide_realpow_zero = thm "LIMSEQ_divide_realpow_zero";
       
  1219 val LIMSEQ_rabs_realpow_zero = thm "LIMSEQ_rabs_realpow_zero";
       
  1220 val NSLIMSEQ_rabs_realpow_zero = thm "NSLIMSEQ_rabs_realpow_zero";
       
  1221 val LIMSEQ_rabs_realpow_zero2 = thm "LIMSEQ_rabs_realpow_zero2";
       
  1222 val NSLIMSEQ_rabs_realpow_zero2 = thm "NSLIMSEQ_rabs_realpow_zero2";
       
  1223 val NSBseq_HFinite_hypreal = thm "NSBseq_HFinite_hypreal";
       
  1224 val NSLIMSEQ_zero_Infinitesimal_hypreal = thm "NSLIMSEQ_zero_Infinitesimal_hypreal";
       
  1225 *}
  1218 *}
  1226 
  1219 
       
  1220 
  1227 end
  1221 end
  1228 
  1222