src/HOL/Complex.thy
changeset 61552 980dd46a03fb
parent 61531 ab2e862263e7
child 61609 77b453bd616f
--- a/src/HOL/Complex.thy	Mon Nov 02 11:56:38 2015 +0100
+++ b/src/HOL/Complex.thy	Mon Nov 02 16:17:09 2015 +0100
@@ -166,6 +166,12 @@
 
 lemma Im_divide_numeral [simp]: "Im (z / numeral w) = Im z / numeral w"
   by (simp add: Im_divide sqr_conv_mult)
+  
+lemma Re_divide_of_nat: "Re (z / of_nat n) = Re z / of_nat n"
+  by (cases n) (simp_all add: Re_divide divide_simps power2_eq_square del: of_nat_Suc)
+
+lemma Im_divide_of_nat: "Im (z / of_nat n) = Im z / of_nat n"
+  by (cases n) (simp_all add: Im_divide divide_simps power2_eq_square del: of_nat_Suc)
 
 lemma of_real_Re [simp]:
     "z \<in> \<real> \<Longrightarrow> of_real (Re z) = z"