src/HOL/Multivariate_Analysis/Linear_Algebra.thy
changeset 62948 7700f467892b
parent 62623 dbc62f86a1a9
child 63007 aa894a49f77d
--- a/src/HOL/Multivariate_Analysis/Linear_Algebra.thy	Sun Apr 10 23:15:34 2016 +0200
+++ b/src/HOL/Multivariate_Analysis/Linear_Algebra.thy	Mon Apr 11 16:27:42 2016 +0100
@@ -784,7 +784,7 @@
   apply (auto simp add: subspace_def)
   done
 
-lemma (in real_vector) independent_empty[intro]: "independent {}"
+lemma (in real_vector) independent_empty [iff]: "independent {}"
   by (simp add: dependent_def)
 
 lemma dependent_single[simp]: "dependent {x} \<longleftrightarrow> x = 0"