src/HOL/Analysis/Inner_Product.thy
changeset 69513 42e08052dae8
parent 69064 5840724b1d71
child 69597 ff784d5a5bfb
--- a/src/HOL/Analysis/Inner_Product.thy	Thu Dec 27 21:32:34 2018 +0100
+++ b/src/HOL/Analysis/Inner_Product.thy	Thu Dec 27 21:32:36 2018 +0100
@@ -177,11 +177,6 @@
   using isCont_power[OF continuous_ident, of x, unfolded isCont_def LIM_eq, rule_format, of e 2]
   by (force simp add: power2_eq_square)
 
-lemma norm_triangle_sub:
-  fixes x y :: "'a::real_normed_vector"
-  shows "norm x \<le> norm y + norm (x - y)"
-  using norm_triangle_ineq[of "y" "x - y"] by (simp add: field_simps)
-
 lemma norm_le: "norm x \<le> norm y \<longleftrightarrow> inner x x \<le> inner y y"
   by (simp add: norm_eq_sqrt_inner)