changeset 15481 | fc075ae929e4 |
parent 15234 | ec91a90c604e |
child 19765 | dfe940911617 |
--- a/src/HOL/Complex/Complex.thy Sun Jan 30 20:48:50 2005 +0100 +++ b/src/HOL/Complex/Complex.thy Tue Feb 01 18:01:57 2005 +0100 @@ -865,9 +865,7 @@ iszero_def) lemma complex_number_of_cnj [simp]: "cnj(number_of v :: complex) = number_of v" -apply (subst complex_number_of [symmetric]) -apply (rule complex_cnj_complex_of_real) -done +by (simp only: complex_number_of [symmetric] complex_cnj_complex_of_real) lemma complex_number_of_cmod: "cmod(number_of v :: complex) = abs (number_of v :: real)"