src/HOL/Real_Asymp/Real_Asymp_Examples.thy
changeset 69597 ff784d5a5bfb
parent 68680 0a0e68369586
child 70817 dd675800469d
equal deleted inserted replaced
69596:c8a2755bf220 69597:ff784d5a5bfb
   229   also have "\<dots> = 2 * sqrt 3" by (subst real_sqrt_mult) simp
   229   also have "\<dots> = 2 * sqrt 3" by (subst real_sqrt_mult) simp
   230   finally show ?thesis by real_asymp
   230   finally show ?thesis by real_asymp
   231 qed
   231 qed
   232 
   232 
   233 
   233 
   234 text \<open>@{url "http://math.stackexchange.com/questions/625574"}\<close>
   234 text \<open>\<^url>\<open>http://math.stackexchange.com/questions/625574\<close>\<close>
   235 lemma "(\<lambda>x::real. (1 - 1/2 * x^2 - cos (x / (1 - x^2))) / x^4) \<midarrow>0\<rightarrow> 23/24"
   235 lemma "(\<lambda>x::real. (1 - 1/2 * x^2 - cos (x / (1 - x^2))) / x^4) \<midarrow>0\<rightarrow> 23/24"
   236   by real_asymp
   236   by real_asymp
   237 
   237 
   238 
   238 
   239 text \<open>@{url "http://math.stackexchange.com/questions/122967"}\<close>
   239 text \<open>\<^url>\<open>http://math.stackexchange.com/questions/122967\<close>\<close>
   240 
   240 
   241 real_limit "\<lambda>x. (x + 1) powr (1 + 1 / x) - x powr (1 + 1 / (x + a))"
   241 real_limit "\<lambda>x. (x + 1) powr (1 + 1 / x) - x powr (1 + 1 / (x + a))"
   242 
   242 
   243 lemma "((\<lambda>x::real. ((x + 1) powr (1 + 1/x) - x powr (1 + 1 / (x + a)))) \<longlongrightarrow> 1) at_top"
   243 lemma "((\<lambda>x::real. ((x + 1) powr (1 + 1/x) - x powr (1 + 1 / (x + a)))) \<longlongrightarrow> 1) at_top"
   244   by real_asymp
   244   by real_asymp
   268 lemma "(\<lambda>x. ((a powr x - x * ln a) / (b powr x - x * ln b)) powr (1 / x ^ 2))
   268 lemma "(\<lambda>x. ((a powr x - x * ln a) / (b powr x - x * ln b)) powr (1 / x ^ 2))
   269          \<midarrow>0\<rightarrow> exp (ln a * ln a / 2 - ln b * ln b / 2)" using ab by real_asymp
   269          \<midarrow>0\<rightarrow> exp (ln a * ln a / 2 - ln b * ln b / 2)" using ab by real_asymp
   270 end
   270 end
   271 
   271 
   272 
   272 
   273 text \<open>@{url "http://math.stackexchange.com/questions/547538"}\<close>
   273 text \<open>\<^url>\<open>http://math.stackexchange.com/questions/547538\<close>\<close>
   274 lemma "(\<lambda>x::real. ((x+4) powr (3/2) + exp x - 9) / x) \<midarrow>0\<rightarrow> 4"
   274 lemma "(\<lambda>x::real. ((x+4) powr (3/2) + exp x - 9) / x) \<midarrow>0\<rightarrow> 4"
   275   by real_asymp
   275   by real_asymp
   276 
   276 
   277 text \<open>@{url "https://www.freemathhelp.com/forum/threads/93513"}\<close>
   277 text \<open>\<^url>\<open>https://www.freemathhelp.com/forum/threads/93513\<close>\<close>
   278 lemma "((\<lambda>x::real. ((3 powr x + 4 powr x) / 4) powr (1/x)) \<longlongrightarrow> 4) at_top"
   278 lemma "((\<lambda>x::real. ((3 powr x + 4 powr x) / 4) powr (1/x)) \<longlongrightarrow> 4) at_top"
   279   by real_asymp
   279   by real_asymp
   280     
   280     
   281 lemma "((\<lambda>x::real. x powr (3/2) * (sqrt (x + 1) + sqrt (x - 1) - 2 * sqrt x)) \<longlongrightarrow> -1/4) at_top"
   281 lemma "((\<lambda>x::real. x powr (3/2) * (sqrt (x + 1) + sqrt (x - 1) - 2 * sqrt x)) \<longlongrightarrow> -1/4) at_top"
   282   by real_asymp
   282   by real_asymp
   283 
   283 
   284 
   284 
   285 text \<open>@{url "https://www.math.ucdavis.edu/~kouba/CalcOneDIRECTORY/limcondirectory/LimitConstant.html"}\<close>
   285 text \<open>\<^url>\<open>https://www.math.ucdavis.edu/~kouba/CalcOneDIRECTORY/limcondirectory/LimitConstant.html\<close>\<close>
   286 lemma  "(\<lambda>x::real. (cos (2*x) - 1) / (cos x - 1)) \<midarrow>0\<rightarrow> 4"
   286 lemma  "(\<lambda>x::real. (cos (2*x) - 1) / (cos x - 1)) \<midarrow>0\<rightarrow> 4"
   287   by real_asymp
   287   by real_asymp
   288 
   288 
   289 lemma "(\<lambda>x::real. tan (2*x) / (x - pi/2)) \<midarrow>pi/2\<rightarrow> 2"
   289 lemma "(\<lambda>x::real. tan (2*x) / (x - pi/2)) \<midarrow>pi/2\<rightarrow> 2"
   290   by real_asymp
   290   by real_asymp
   292 
   292 
   293 text \<open>@url{"https://www.math.ucdavis.edu/~kouba/CalcOneDIRECTORY/liminfdirectory/LimitInfinity.html"}\<close>
   293 text \<open>@url{"https://www.math.ucdavis.edu/~kouba/CalcOneDIRECTORY/liminfdirectory/LimitInfinity.html"}\<close>
   294 lemma "filterlim (\<lambda>x::real. (3 powr x + 3 powr (2*x)) powr (1/x)) (nhds 9) at_top"
   294 lemma "filterlim (\<lambda>x::real. (3 powr x + 3 powr (2*x)) powr (1/x)) (nhds 9) at_top"
   295   using powr_def[of 3 "2::real"] by real_asymp
   295   using powr_def[of 3 "2::real"] by real_asymp
   296 
   296 
   297 text \<open>@{url "https://www.math.ucdavis.edu/~kouba/CalcOneDIRECTORY/lhopitaldirectory/LHopital.html"}\<close>
   297 text \<open>\<^url>\<open>https://www.math.ucdavis.edu/~kouba/CalcOneDIRECTORY/lhopitaldirectory/LHopital.html\<close>\<close>
   298 lemma "filterlim (\<lambda>x::real. (x^2 - 1) / (x^2 + 3*x - 4)) (nhds (2/5)) (at 1)"
   298 lemma "filterlim (\<lambda>x::real. (x^2 - 1) / (x^2 + 3*x - 4)) (nhds (2/5)) (at 1)"
   299   by real_asymp
   299   by real_asymp
   300     
   300     
   301 lemma "filterlim (\<lambda>x::real. (x - 4) / (sqrt x - 2)) (nhds 4) (at 4)"
   301 lemma "filterlim (\<lambda>x::real. (x - 4) / (sqrt x - 2)) (nhds 4) (at 4)"
   302   by real_asymp
   302   by real_asymp
   373 
   373 
   374 lemma "filterlim (\<lambda>x::real. x powr (x powr x)) (at_right 0) (at_right 0)"
   374 lemma "filterlim (\<lambda>x::real. x powr (x powr x)) (at_right 0) (at_right 0)"
   375   by (real_asymp (verbose))
   375   by (real_asymp (verbose))
   376 
   376 
   377 
   377 
   378 text \<open>@{url "http://calculus.nipissingu.ca/problems/limit_problems.html"}\<close>
   378 text \<open>\<^url>\<open>http://calculus.nipissingu.ca/problems/limit_problems.html\<close>\<close>
   379 lemma "((\<lambda>x::real. (x^2 - 1) / \<bar>x - 1\<bar>) \<longlongrightarrow> -2) (at_left 1)"
   379 lemma "((\<lambda>x::real. (x^2 - 1) / \<bar>x - 1\<bar>) \<longlongrightarrow> -2) (at_left 1)"
   380       "((\<lambda>x::real. (x^2 - 1) / \<bar>x - 1\<bar>) \<longlongrightarrow> 2) (at_right 1)"
   380       "((\<lambda>x::real. (x^2 - 1) / \<bar>x - 1\<bar>) \<longlongrightarrow> 2) (at_right 1)"
   381   by real_asymp+
   381   by real_asymp+
   382 
   382 
   383 lemma "((\<lambda>x::real. (root 3 x - 1) / \<bar>sqrt x - 1\<bar>) \<longlongrightarrow> -2 / 3) (at_left 1)"
   383 lemma "((\<lambda>x::real. (root 3 x - 1) / \<bar>sqrt x - 1\<bar>) \<longlongrightarrow> -2 / 3) (at_left 1)"
   384       "((\<lambda>x::real. (root 3 x - 1) / \<bar>sqrt x - 1\<bar>) \<longlongrightarrow> 2 / 3) (at_right 1)"
   384       "((\<lambda>x::real. (root 3 x - 1) / \<bar>sqrt x - 1\<bar>) \<longlongrightarrow> 2 / 3) (at_right 1)"
   385   by real_asymp+
   385   by real_asymp+
   386 
   386 
   387 
   387 
   388 text \<open>@{url "https://math.stackexchange.com/questions/547538"}\<close>
   388 text \<open>\<^url>\<open>https://math.stackexchange.com/questions/547538\<close>\<close>
   389 
   389 
   390 lemma "(\<lambda>x::real. ((x + 4) powr (3/2) + exp x - 9) / x) \<midarrow>0\<rightarrow> 4"
   390 lemma "(\<lambda>x::real. ((x + 4) powr (3/2) + exp x - 9) / x) \<midarrow>0\<rightarrow> 4"
   391   by real_asymp
   391   by real_asymp
   392 
   392 
   393 text \<open>@{url "https://math.stackexchange.com/questions/625574"}\<close>
   393 text \<open>\<^url>\<open>https://math.stackexchange.com/questions/625574\<close>\<close>
   394 lemma "(\<lambda>x::real. (1 - x^2 / 2 - cos (x / (1 - x^2))) / x^4) \<midarrow>0\<rightarrow> 23/24"
   394 lemma "(\<lambda>x::real. (1 - x^2 / 2 - cos (x / (1 - x^2))) / x^4) \<midarrow>0\<rightarrow> 23/24"
   395   by real_asymp
   395   by real_asymp
   396 
   396 
   397 text \<open>@{url "https://www.mapleprimes.com/questions/151308-A-Hard-Limit-Question"}\<close>
   397 text \<open>\<^url>\<open>https://www.mapleprimes.com/questions/151308-A-Hard-Limit-Question\<close>\<close>
   398 lemma "(\<lambda>x::real. x / (x - 1) - 1 / ln x) \<midarrow>1\<rightarrow> 1 / 2"
   398 lemma "(\<lambda>x::real. x / (x - 1) - 1 / ln x) \<midarrow>1\<rightarrow> 1 / 2"
   399   by real_asymp
   399   by real_asymp
   400 
   400 
   401 text \<open>@{url "https://www.freemathhelp.com/forum/threads/93513-two-extremely-difficult-limit-problems"}\<close>
   401 text \<open>\<^url>\<open>https://www.freemathhelp.com/forum/threads/93513-two-extremely-difficult-limit-problems\<close>\<close>
   402 lemma "((\<lambda>x::real. ((3 powr x + 4 powr x) / 4) powr (1/x)) \<longlongrightarrow> 4) at_top"
   402 lemma "((\<lambda>x::real. ((3 powr x + 4 powr x) / 4) powr (1/x)) \<longlongrightarrow> 4) at_top"
   403   by real_asymp
   403   by real_asymp
   404 
   404 
   405 lemma "((\<lambda>x::real. x powr 1.5 * (sqrt (x + 1) + sqrt (x - 1) - 2 * sqrt x)) \<longlongrightarrow> -1/4) at_top"
   405 lemma "((\<lambda>x::real. x powr 1.5 * (sqrt (x + 1) + sqrt (x - 1) - 2 * sqrt x)) \<longlongrightarrow> -1/4) at_top"
   406   by real_asymp
   406   by real_asymp
   407 
   407 
   408 text \<open>@{url "https://math.stackexchange.com/questions/1390833"}\<close>
   408 text \<open>\<^url>\<open>https://math.stackexchange.com/questions/1390833\<close>\<close>
   409 context
   409 context
   410   fixes a b :: real
   410   fixes a b :: real
   411   assumes ab: "a + b > 0" "a + b = 1"
   411   assumes ab: "a + b > 0" "a + b = 1"
   412 begin
   412 begin
   413 real_limit "\<lambda>x. (a * x powr (1 / x) + b) powr (x / ln x)"
   413 real_limit "\<lambda>x. (a * x powr (1 / x) + b) powr (x / ln x)"