src/HOL/NthRoot.thy
changeset 63721 492bb53c3420
parent 63558 0aa33085c8b1
child 64122 74fde524799e
--- a/src/HOL/NthRoot.thy	Wed Aug 24 11:02:23 2016 +0200
+++ b/src/HOL/NthRoot.thy	Thu Aug 25 15:50:43 2016 +0200
@@ -469,6 +469,14 @@
 lemma real_less_rsqrt: "x\<^sup>2 < y \<Longrightarrow> x < sqrt y"
   using real_sqrt_less_mono[of "x\<^sup>2" y] by simp
 
+lemma real_sqrt_power_even: 
+  assumes "even n" "x \<ge> 0"
+  shows   "sqrt x ^ n = x ^ (n div 2)"
+proof -
+  from assms obtain k where "n = 2*k" by (auto elim!: evenE)
+  with assms show ?thesis by (simp add: power_mult)
+qed
+
 lemma sqrt_le_D: "sqrt x \<le> y \<Longrightarrow> x \<le> y\<^sup>2"
   by (meson not_le real_less_rsqrt)