src/HOL/Complex.thy
changeset 64290 fb5c74a58796
parent 64272 f76b6dda2e56
child 64773 223b2ebdda79
--- a/src/HOL/Complex.thy	Tue Oct 18 17:29:28 2016 +0200
+++ b/src/HOL/Complex.thy	Tue Oct 18 18:48:53 2016 +0200
@@ -381,6 +381,23 @@
   by (simp add: complex_sgn_def divide_inverse)
 
 
+subsection \<open>Absolute value\<close>
+
+instantiation complex :: field_abs_sgn
+begin
+
+definition abs_complex :: "complex \<Rightarrow> complex"
+  where "abs_complex = of_real \<circ> norm"
+
+instance
+  apply standard
+         apply (auto simp add: abs_complex_def complex_sgn_def norm_mult)
+  apply (auto simp add: scaleR_conv_of_real field_simps)
+  done
+
+end
+
+
 subsection \<open>Completeness of the Complexes\<close>
 
 lemma bounded_linear_Re: "bounded_linear Re"