src/HOL/Log.thy
changeset 50346 a75c6429c3c3
parent 50322 b06b95a5fda2
child 51478 270b21f3ae0a
equal deleted inserted replaced
50345:8cf33d605e81 50346:a75c6429c3c3
   362   assumes "s < 0" and "LIM x F. f x :> at_top"
   362   assumes "s < 0" and "LIM x F. f x :> at_top"
   363   shows "((\<lambda>x. f x powr s) ---> 0) F"
   363   shows "((\<lambda>x. f x powr s) ---> 0) F"
   364 proof (rule tendstoI)
   364 proof (rule tendstoI)
   365   fix e :: real assume "0 < e"
   365   fix e :: real assume "0 < e"
   366   def Z \<equiv> "e powr (1 / s)"
   366   def Z \<equiv> "e powr (1 / s)"
   367   from assms have "eventually (\<lambda>x. Z < f x) F" by (simp add: filterlim_at_top)
   367   from assms have "eventually (\<lambda>x. Z < f x) F"
       
   368     by (simp add: filterlim_at_top_dense)
   368   moreover
   369   moreover
   369   from assms have "\<And>x. Z < x \<Longrightarrow> x powr s < Z powr s"
   370   from assms have "\<And>x. Z < x \<Longrightarrow> x powr s < Z powr s"
   370     by (auto simp: Z_def intro!: powr_less_mono2_neg)
   371     by (auto simp: Z_def intro!: powr_less_mono2_neg)
   371   with assms `0 < e` have "\<And>x. Z < x \<Longrightarrow> dist (x powr s) 0 < e"
   372   with assms `0 < e` have "\<And>x. Z < x \<Longrightarrow> dist (x powr s) 0 < e"
   372     by (simp add: powr_powr Z_def dist_real_def)
   373     by (simp add: powr_powr Z_def dist_real_def)