src/HOL/Hyperreal/Lim.thy
changeset 23127 56ee8105c002
parent 23118 ce3cf072ae14
child 23441 ee218296d635
equal deleted inserted replaced
23126:93f8cb025afd 23127:56ee8105c002
   369 apply (erule (1) LIM_prod_zero)
   369 apply (erule (1) LIM_prod_zero)
   370 apply (erule LIM_left_zero)
   370 apply (erule LIM_left_zero)
   371 apply (erule LIM_right_zero)
   371 apply (erule LIM_right_zero)
   372 done
   372 done
   373 
   373 
   374 lemmas LIM_mult = bounded_bilinear_mult.LIM
   374 lemmas LIM_mult = mult.LIM
   375 
   375 
   376 lemmas LIM_mult_zero = bounded_bilinear_mult.LIM_prod_zero
   376 lemmas LIM_mult_zero = mult.LIM_prod_zero
   377 
   377 
   378 lemmas LIM_mult_left_zero = bounded_bilinear_mult.LIM_left_zero
   378 lemmas LIM_mult_left_zero = mult.LIM_left_zero
   379 
   379 
   380 lemmas LIM_mult_right_zero = bounded_bilinear_mult.LIM_right_zero
   380 lemmas LIM_mult_right_zero = mult.LIM_right_zero
   381 
   381 
   382 lemmas LIM_scaleR = bounded_bilinear_scaleR.LIM
   382 lemmas LIM_scaleR = scaleR.LIM
   383 
   383 
   384 lemmas LIM_of_real = bounded_linear_of_real.LIM
   384 lemmas LIM_of_real = of_real.LIM
   385 
   385 
   386 lemma LIM_power:
   386 lemma LIM_power:
   387   fixes f :: "'a::real_normed_vector \<Rightarrow> 'b::{recpower,real_normed_algebra}"
   387   fixes f :: "'a::real_normed_vector \<Rightarrow> 'b::{recpower,real_normed_algebra}"
   388   assumes f: "f -- a --> l"
   388   assumes f: "f -- a --> l"
   389   shows "(\<lambda>x. f x ^ n) -- a --> l ^ n"
   389   shows "(\<lambda>x. f x ^ n) -- a --> l ^ n"
   517 
   517 
   518 lemma (in bounded_bilinear) isCont:
   518 lemma (in bounded_bilinear) isCont:
   519   "\<lbrakk>isCont f a; isCont g a\<rbrakk> \<Longrightarrow> isCont (\<lambda>x. f x ** g x) a"
   519   "\<lbrakk>isCont f a; isCont g a\<rbrakk> \<Longrightarrow> isCont (\<lambda>x. f x ** g x) a"
   520   unfolding isCont_def by (rule LIM)
   520   unfolding isCont_def by (rule LIM)
   521 
   521 
   522 lemmas isCont_scaleR = bounded_bilinear_scaleR.isCont
   522 lemmas isCont_scaleR = scaleR.isCont
   523 
   523 
   524 lemma isCont_of_real:
   524 lemma isCont_of_real:
   525   "isCont f a \<Longrightarrow> isCont (\<lambda>x. of_real (f x)) a"
   525   "isCont f a \<Longrightarrow> isCont (\<lambda>x. of_real (f x)) a"
   526   unfolding isCont_def by (rule LIM_of_real)
   526   unfolding isCont_def by (rule LIM_of_real)
   527 
   527