src/HOL/Real_Asymp/Real_Asymp_Examples.thy
changeset 68680 0a0e68369586
parent 68630 c55f6f0b3854
child 69597 ff784d5a5bfb
equal deleted inserted replaced
68679:2a20b315a44d 68680:0a0e68369586
    98   shows   "(f \<longlongrightarrow> 0) at_top" (is ?thesis1)
    98   shows   "(f \<longlongrightarrow> 0) at_top" (is ?thesis1)
    99           "f \<sim> (\<lambda>x. -(ln x ^ 2) / (2*x))" (is ?thesis2)
    99           "f \<sim> (\<lambda>x. -(ln x ^ 2) / (2*x))" (is ?thesis2)
   100   unfolding f_def by real_asymp+
   100   unfolding f_def by real_asymp+
   101 
   101 
   102   
   102   
   103 subsection \<open>Asymptotic inequalities related to the Akra–Bazzi theorem\<close>
   103 subsection \<open>Asymptotic inequalities related to the Akra--Bazzi theorem\<close>
   104   
   104   
   105 definition "akra_bazzi_asymptotic1 b hb e p x \<longleftrightarrow>
   105 definition "akra_bazzi_asymptotic1 b hb e p x \<longleftrightarrow>
   106   (1 - hb * inverse b * ln x powr -(1+e)) powr p * (1 + ln (b*x + hb*x/ln x powr (1+e)) powr (-e/2))
   106   (1 - hb * inverse b * ln x powr -(1+e)) powr p * (1 + ln (b*x + hb*x/ln x powr (1+e)) powr (-e/2))
   107   \<ge> 1 + (ln x powr (-e/2) :: real)"
   107   \<ge> 1 + (ln x powr (-e/2) :: real)"
   108 definition "akra_bazzi_asymptotic1' b hb e p x \<longleftrightarrow>
   108 definition "akra_bazzi_asymptotic1' b hb e p x \<longleftrightarrow>