src/HOL/Complex.thy
changeset 59862 44b3f4fa33ca
parent 59746 ddae5727c5a9
child 59867 58043346ca64
--- a/src/HOL/Complex.thy	Tue Mar 31 00:21:07 2015 +0200
+++ b/src/HOL/Complex.thy	Tue Mar 31 15:00:03 2015 +0100
@@ -93,10 +93,10 @@
 lemma Im_power2: "Im (x ^ 2) = 2 * Re x * Im x"
   by (simp add: power2_eq_square)
 
-lemma Re_power_real: "Im x = 0 \<Longrightarrow> Re (x ^ n) = Re x ^ n "
+lemma Re_power_real [simp]: "Im x = 0 \<Longrightarrow> Re (x ^ n) = Re x ^ n "
   by (induct n) simp_all
 
-lemma Im_power_real: "Im x = 0 \<Longrightarrow> Im (x ^ n) = 0"
+lemma Im_power_real [simp]: "Im x = 0 \<Longrightarrow> Im (x ^ n) = 0"
   by (induct n) simp_all
 
 subsection {* Scalar Multiplication *}
@@ -823,6 +823,9 @@
 lemma csqrt_of_real_nonpos [simp]: "Im x = 0 \<Longrightarrow> Re x \<le> 0 \<Longrightarrow> csqrt x = \<i> * sqrt \<bar>Re x\<bar>"
   by (simp add: complex_eq_iff norm_complex_def)
 
+lemma of_real_sqrt: "x \<ge> 0 \<Longrightarrow> of_real (sqrt x) = csqrt (of_real x)"
+  by (simp add: complex_eq_iff norm_complex_def)
+
 lemma csqrt_0 [simp]: "csqrt 0 = 0"
   by simp