src/HOL/Real_Vector_Spaces.thy
changeset 54230 b1d955791529
parent 53600 8fda7ad57466
child 54263 c4159fe6fa46
--- a/src/HOL/Real_Vector_Spaces.thy	Thu Oct 31 16:54:22 2013 +0100
+++ b/src/HOL/Real_Vector_Spaces.thy	Fri Nov 01 18:51:14 2013 +0100
@@ -31,7 +31,7 @@
 qed
 
 lemma diff: "f (x - y) = f x - f y"
-by (simp add: add minus diff_minus)
+  using add [of x "- y"] by (simp add: minus)
 
 lemma setsum: "f (setsum g A) = (\<Sum>x\<in>A. f (g x))"
 apply (cases "finite A")
@@ -553,8 +553,7 @@
 proof -
   have "norm (a + - b) \<le> norm a + norm (- b)"
     by (rule norm_triangle_ineq)
-  thus ?thesis
-    by (simp only: diff_minus norm_minus_cancel)
+  then show ?thesis by simp
 qed
 
 lemma norm_diff_ineq:
@@ -571,7 +570,7 @@
   shows "norm ((a + b) - (c + d)) \<le> norm (a - c) + norm (b - d)"
 proof -
   have "norm ((a + b) - (c + d)) = norm ((a - c) + (b - d))"
-    by (simp add: diff_minus add_ac)
+    by (simp add: algebra_simps)
   also have "\<dots> \<le> norm (a - c) + norm (b - d)"
     by (rule norm_triangle_ineq)
   finally show ?thesis .