src/HOL/Analysis/Convex_Euclidean_Space.thy
changeset 63945 444eafb6e864
parent 63938 f6ce08859d4c
child 63955 51a3d38d2281
--- a/src/HOL/Analysis/Convex_Euclidean_Space.thy	Mon Sep 26 16:57:05 2016 +0200
+++ b/src/HOL/Analysis/Convex_Euclidean_Space.thy	Tue Sep 27 16:24:53 2016 +0100
@@ -7748,6 +7748,22 @@
     using rel_interior_empty by auto
 qed
 
+lemma interior_simplex_nonempty:
+  fixes S :: "'N :: euclidean_space set"
+  assumes "independent S" "finite S" "card S = DIM('N)"
+  obtains a where "a \<in> interior (convex hull (insert 0 S))"
+proof -
+  have "affine hull (insert 0 S) = UNIV"
+    apply (simp add: hull_inc affine_hull_span_0)
+    using assms dim_eq_full indep_card_eq_dim_span by fastforce
+  moreover have "rel_interior (convex hull insert 0 S) \<noteq> {}"
+    using rel_interior_eq_empty [of "convex hull (insert 0 S)"] by auto
+  ultimately have "interior (convex hull insert 0 S) \<noteq> {}"
+    by (simp add: rel_interior_interior)
+  with that show ?thesis
+    by auto
+qed
+
 lemma convex_rel_interior:
   fixes S :: "'n::euclidean_space set"
   assumes "convex S"