src/HOL/Log.thy
changeset 45930 2a882ef2cd73
parent 45916 758671e966a0
child 47593 69f0af2b7d54
--- a/src/HOL/Log.thy	Mon Dec 19 13:58:54 2011 +0100
+++ b/src/HOL/Log.thy	Mon Dec 19 14:41:08 2011 +0100
@@ -60,6 +60,10 @@
 lemma powr_add: "x powr (a + b) = (x powr a) * (x powr b)"
 by (simp add: powr_def exp_add [symmetric] left_distrib)
 
+lemma powr_mult_base:
+  "0 < x \<Longrightarrow>x * x powr y = x powr (1 + y)"
+using assms by (auto simp: powr_add)
+
 lemma powr_powr: "(x powr a) powr b = x powr (a * b)"
 by (simp add: powr_def)
 
@@ -178,6 +182,10 @@
   apply (rule powr_realpow [THEN sym], simp)
 done
 
+lemma root_powr_inverse:
+  "0 < n \<Longrightarrow> 0 < x \<Longrightarrow> root n x = x powr (1/n)"
+by (auto simp: root_def powr_realpow[symmetric] powr_powr)
+
 lemma ln_powr: "0 < x ==> 0 < y ==> ln(x powr y) = y * ln x"
 by (unfold powr_def, simp)