src/HOL/Analysis/Inner_Product.thy
changeset 68499 d4312962161a
parent 68073 fad29d2a17a5
child 68611 4bc4b5c0ccfc
--- a/src/HOL/Analysis/Inner_Product.thy	Mon Jun 25 14:06:50 2018 +0100
+++ b/src/HOL/Analysis/Inner_Product.thy	Tue Jun 26 14:51:18 2018 +0100
@@ -322,9 +322,9 @@
     unfolding inner_complex_def by simp
   show "inner x x = 0 \<longleftrightarrow> x = 0"
     unfolding inner_complex_def
-    by (simp add: add_nonneg_eq_0_iff complex_Re_Im_cancel_iff)
+    by (simp add: add_nonneg_eq_0_iff complex_eq_iff)
   show "norm x = sqrt (inner x x)"
-    unfolding inner_complex_def complex_norm_def
+    unfolding inner_complex_def norm_complex_def
     by (simp add: power2_eq_square)
 qed