declare complex_diff as simp rule
authorhuffman
Wed, 06 Jun 2007 16:42:39 +0200
changeset 23275 339cdc29b0bc
parent 23274 f997514ad8f4
child 23276 a70934b63910
declare complex_diff as simp rule
src/HOL/Complex/Complex.thy
--- a/src/HOL/Complex/Complex.thy	Wed Jun 06 16:12:08 2007 +0200
+++ b/src/HOL/Complex/Complex.thy	Wed Jun 06 16:42:39 2007 +0200
@@ -75,7 +75,7 @@
 lemma complex_Im_minus [simp]: "Im (- x) = - Im x"
 by (simp add: complex_minus_def)
 
-lemma complex_diff:
+lemma complex_diff [simp]:
   "Complex a b - Complex c d = Complex (a - c) (b - d)"
 by (simp add: complex_diff_def)
 
@@ -363,7 +363,6 @@
 apply (drule_tac r="r / sqrt 2" in LIMSEQ_D, safe)
 apply (drule_tac r="r / sqrt 2" in LIMSEQ_D, safe)
 apply (rename_tac M N, rule_tac x="max M N" in exI, safe)
-apply (simp add: complex_diff)
 apply (simp add: real_sqrt_sum_squares_less)
 apply (simp add: divide_pos_pos)
 done