src/HOL/Multivariate_Analysis/Linear_Algebra.thy
changeset 60162 645058aa9d6f
parent 60150 bd773c47ad0b
child 60303 00c06f1315d0
--- a/src/HOL/Multivariate_Analysis/Linear_Algebra.thy	Wed Apr 29 14:04:22 2015 +0100
+++ b/src/HOL/Multivariate_Analysis/Linear_Algebra.thy	Thu Apr 30 15:28:01 2015 +0100
@@ -575,9 +575,8 @@
     by simp
   also have "\<dots> \<le> (1 + x) ^ Suc n"
     apply (subst diff_le_0_iff_le[symmetric])
+    using mult_left_mono[OF p Suc.prems]
     apply (simp add: field_simps)
-    using mult_left_mono[OF p Suc.prems]
-    apply simp
     done
   finally show ?case
     by (simp add: real_of_nat_Suc field_simps)
@@ -887,10 +886,8 @@
   assumes "0 \<in> A"
   shows "dependent A"
   unfolding dependent_def
-  apply (rule_tac x=0 in bexI)
   using assms span_0
-  apply auto
-  done
+  by auto
 
 lemma (in real_vector) span_add: "x \<in> span S \<Longrightarrow> y \<in> span S \<Longrightarrow> x + y \<in> span S"
   by (metis subspace_add subspace_span)