diff -r 2a74926bd760 -r bbe2730e6db6 src/HOL/Multivariate_Analysis/Vec1.thy --- a/src/HOL/Multivariate_Analysis/Vec1.thy Mon Apr 26 15:51:10 2010 -0700 +++ b/src/HOL/Multivariate_Analysis/Vec1.thy Mon Apr 26 16:28:58 2010 -0700 @@ -394,6 +394,11 @@ hence "\K. \x. \f x\ \ \x\ * K" apply(rule_tac x=K in exI) unfolding vec1_dest_vec1_simps by (auto simp add:field_simps) } thus ?thesis unfolding linear_def bounded_linear_def additive_def bounded_linear_axioms_def o_def - unfolding vec1_dest_vec1_simps by auto qed + unfolding vec1_dest_vec1_simps by auto qed + +lemma vec1_le[simp]:fixes a::real shows "vec1 a \ vec1 b \ a \ b" + unfolding vector_le_def by auto +lemma vec1_less[simp]:fixes a::real shows "vec1 a < vec1 b \ a < b" + unfolding vector_less_def by auto end