src/HOL/Real_Vector_Spaces.thy
changeset 61762 d50b993b4fb9
parent 61649 268d88ec9087
child 61799 4cf66f21b764
--- a/src/HOL/Real_Vector_Spaces.thy	Mon Nov 30 14:24:51 2015 +0100
+++ b/src/HOL/Real_Vector_Spaces.thy	Tue Dec 01 14:09:10 2015 +0000
@@ -9,6 +9,10 @@
 imports Real Topological_Spaces
 begin
 
+
+lemma (in ordered_ab_group_add) diff_ge_0_iff_ge [simp]: "a - b \<ge> 0 \<longleftrightarrow> a \<ge> b"
+  by (simp add: le_diff_eq)
+
 subsection \<open>Locale for additive functions\<close>
 
 locale additive =
@@ -777,6 +781,11 @@
   thus ?thesis by simp
 qed
 
+lemma norm_add_leD:
+  fixes a b :: "'a::real_normed_vector"
+  shows "norm (a + b) \<le> c \<Longrightarrow> norm b \<le> norm a + c"
+    by (metis add.commute diff_le_eq norm_diff_ineq order.trans)
+
 lemma norm_diff_triangle_ineq:
   fixes a b c d :: "'a::real_normed_vector"
   shows "norm ((a + b) - (c + d)) \<le> norm (a - c) + norm (b - d)"