src/HOL/Real_Vector_Spaces.thy
changeset 61762 d50b993b4fb9
parent 61649 268d88ec9087
child 61799 4cf66f21b764
equal deleted inserted replaced
61757:0d399131008f 61762:d50b993b4fb9
     6 section \<open>Vector Spaces and Algebras over the Reals\<close>
     6 section \<open>Vector Spaces and Algebras over the Reals\<close>
     7 
     7 
     8 theory Real_Vector_Spaces
     8 theory Real_Vector_Spaces
     9 imports Real Topological_Spaces
     9 imports Real Topological_Spaces
    10 begin
    10 begin
       
    11 
       
    12 
       
    13 lemma (in ordered_ab_group_add) diff_ge_0_iff_ge [simp]: "a - b \<ge> 0 \<longleftrightarrow> a \<ge> b"
       
    14   by (simp add: le_diff_eq)
    11 
    15 
    12 subsection \<open>Locale for additive functions\<close>
    16 subsection \<open>Locale for additive functions\<close>
    13 
    17 
    14 locale additive =
    18 locale additive =
    15   fixes f :: "'a::ab_group_add \<Rightarrow> 'b::ab_group_add"
    19   fixes f :: "'a::ab_group_add \<Rightarrow> 'b::ab_group_add"
   774 proof -
   778 proof -
   775   have "norm a - norm (- b) \<le> norm (a - - b)"
   779   have "norm a - norm (- b) \<le> norm (a - - b)"
   776     by (rule norm_triangle_ineq2)
   780     by (rule norm_triangle_ineq2)
   777   thus ?thesis by simp
   781   thus ?thesis by simp
   778 qed
   782 qed
       
   783 
       
   784 lemma norm_add_leD:
       
   785   fixes a b :: "'a::real_normed_vector"
       
   786   shows "norm (a + b) \<le> c \<Longrightarrow> norm b \<le> norm a + c"
       
   787     by (metis add.commute diff_le_eq norm_diff_ineq order.trans)
   779 
   788 
   780 lemma norm_diff_triangle_ineq:
   789 lemma norm_diff_triangle_ineq:
   781   fixes a b c d :: "'a::real_normed_vector"
   790   fixes a b c d :: "'a::real_normed_vector"
   782   shows "norm ((a + b) - (c + d)) \<le> norm (a - c) + norm (b - d)"
   791   shows "norm ((a + b) - (c + d)) \<le> norm (a - c) + norm (b - d)"
   783 proof -
   792 proof -