src/HOL/Lim.thy
changeset 44282 f0de18b62d63
parent 44254 336dd390e4a4
child 44310 ba3d031b5dbb
equal deleted inserted replaced
44275:d995733b635d 44282:f0de18b62d63
   319 
   319 
   320 lemma (in bounded_bilinear) LIM_right_zero:
   320 lemma (in bounded_bilinear) LIM_right_zero:
   321   "f -- a --> 0 \<Longrightarrow> (\<lambda>x. c ** f x) -- a --> 0"
   321   "f -- a --> 0 \<Longrightarrow> (\<lambda>x. c ** f x) -- a --> 0"
   322   by (rule tendsto_right_zero)
   322   by (rule tendsto_right_zero)
   323 
   323 
   324 lemmas LIM_mult = mult.LIM
   324 lemmas LIM_mult =
   325 
   325   bounded_bilinear.LIM [OF bounded_bilinear_mult]
   326 lemmas LIM_mult_zero = mult.LIM_prod_zero
   326 
   327 
   327 lemmas LIM_mult_zero =
   328 lemmas LIM_mult_left_zero = mult.LIM_left_zero
   328   bounded_bilinear.LIM_prod_zero [OF bounded_bilinear_mult]
   329 
   329 
   330 lemmas LIM_mult_right_zero = mult.LIM_right_zero
   330 lemmas LIM_mult_left_zero =
   331 
   331   bounded_bilinear.LIM_left_zero [OF bounded_bilinear_mult]
   332 lemmas LIM_scaleR = scaleR.LIM
   332 
   333 
   333 lemmas LIM_mult_right_zero =
   334 lemmas LIM_of_real = of_real.LIM
   334   bounded_bilinear.LIM_right_zero [OF bounded_bilinear_mult]
       
   335 
       
   336 lemmas LIM_scaleR =
       
   337   bounded_bilinear.LIM [OF bounded_bilinear_scaleR]
       
   338 
       
   339 lemmas LIM_of_real =
       
   340   bounded_linear.LIM [OF bounded_linear_of_real]
   335 
   341 
   336 lemma LIM_power:
   342 lemma LIM_power:
   337   fixes f :: "'a::topological_space \<Rightarrow> 'b::{power,real_normed_algebra}"
   343   fixes f :: "'a::topological_space \<Rightarrow> 'b::{power,real_normed_algebra}"
   338   assumes f: "f -- a --> l"
   344   assumes f: "f -- a --> l"
   339   shows "(\<lambda>x. f x ^ n) -- a --> l ^ n"
   345   shows "(\<lambda>x. f x ^ n) -- a --> l ^ n"
   444 
   450 
   445 lemma (in bounded_bilinear) isCont:
   451 lemma (in bounded_bilinear) isCont:
   446   "\<lbrakk>isCont f a; isCont g a\<rbrakk> \<Longrightarrow> isCont (\<lambda>x. f x ** g x) a"
   452   "\<lbrakk>isCont f a; isCont g a\<rbrakk> \<Longrightarrow> isCont (\<lambda>x. f x ** g x) a"
   447   unfolding isCont_def by (rule LIM)
   453   unfolding isCont_def by (rule LIM)
   448 
   454 
   449 lemmas isCont_scaleR [simp] = scaleR.isCont
   455 lemmas isCont_scaleR [simp] =
   450 
   456   bounded_bilinear.isCont [OF bounded_bilinear_scaleR]
   451 lemma isCont_of_real [simp]:
   457 
   452   "isCont f a \<Longrightarrow> isCont (\<lambda>x. of_real (f x)::'b::real_normed_algebra_1) a"
   458 lemmas isCont_of_real [simp] =
   453   by (rule of_real.isCont)
   459   bounded_linear.isCont [OF bounded_linear_of_real]
   454 
   460 
   455 lemma isCont_power [simp]:
   461 lemma isCont_power [simp]:
   456   fixes f :: "'a::topological_space \<Rightarrow> 'b::{power,real_normed_algebra}"
   462   fixes f :: "'a::topological_space \<Rightarrow> 'b::{power,real_normed_algebra}"
   457   shows "isCont f a \<Longrightarrow> isCont (\<lambda>x. f x ^ n) a"
   463   shows "isCont f a \<Longrightarrow> isCont (\<lambda>x. f x ^ n) a"
   458   unfolding isCont_def by (rule LIM_power)
   464   unfolding isCont_def by (rule LIM_power)