src/HOL/Complex.thy
changeset 44842 282eef2c0f77
parent 44841 e55503200061
child 44843 93d0f85cfe4a
--- a/src/HOL/Complex.thy	Thu Sep 08 07:06:59 2011 -0700
+++ b/src/HOL/Complex.thy	Thu Sep 08 07:16:47 2011 -0700
@@ -549,12 +549,6 @@
 lemma Im_sgn [simp]: "Im(sgn z) = Im(z)/cmod z"
   by (simp add: complex_sgn_def divide_inverse)
 
-lemma complex_inverse_complex_split:
-     "inverse(complex_of_real x + ii * complex_of_real y) =
-      complex_of_real(x/(x ^ 2 + y ^ 2)) -
-      ii * complex_of_real(y/(x ^ 2 + y ^ 2))"
-  by (simp add: complex_of_real_def i_def diff_minus divide_inverse)
-
 (*----------------------------------------------------------------------------*)
 (* Many of the theorems below need to be moved elsewhere e.g. Transc. Also *)
 (* many of the theorems are not used - so should they be kept?                *)