src/HOL/Log.thy
changeset 45915 0e5a87b772f9
parent 45892 8dcf6692433f
child 45916 758671e966a0
--- a/src/HOL/Log.thy	Sun Dec 18 14:28:14 2011 +0100
+++ b/src/HOL/Log.thy	Thu Dec 15 17:21:29 2011 +0100
@@ -285,6 +285,10 @@
   finally show ?thesis .
 qed
 
+lemma tendsto_powr [tendsto_intros]:
+  "\<lbrakk>(f ---> a) F; (g ---> b) F; 0 < a\<rbrakk> \<Longrightarrow> ((\<lambda>x. f x powr g x) ---> a powr b) F"
+  unfolding powr_def by (intro tendsto_intros)
+
 (* FIXME: generalize by replacing d by with g x and g ---> d? *)
 lemma tendsto_zero_powrI:
   assumes "eventually (\<lambda>x. 0 < f x ) F" and "(f ---> 0) F"