src/HOL/Analysis/Starlike.thy
changeset 71240 67880e7ee08d
parent 71236 6c1ed478605e
child 71244 38457af660bc
--- a/src/HOL/Analysis/Starlike.thy	Thu Dec 05 13:51:09 2019 +0100
+++ b/src/HOL/Analysis/Starlike.thy	Thu Dec 05 18:26:11 2019 +0100
@@ -3842,9 +3842,6 @@
     by (simp add: collinear_subset)
 qed
 
-lemma affine_hull_eq_empty [simp]: "affine hull S = {} \<longleftrightarrow> S = {}"
-  using affine_hull_nonempty by blast
-
 lemma affine_hull_2_alt:
   fixes a b :: "'a::real_vector"
   shows "affine hull {a,b} = range (\<lambda>u. a + u *\<^sub>R (b - a))"