src/HOL/Library/Convex.thy
changeset 53596 d29d63460d84
parent 51642 400ec5ae7f8f
child 53620 3c7f5e7926dc
--- a/src/HOL/Library/Convex.thy	Thu Sep 12 09:06:46 2013 -0700
+++ b/src/HOL/Library/Convex.thy	Thu Sep 12 09:33:36 2013 -0700
@@ -46,6 +46,12 @@
 lemma convex_Int: "convex s \<Longrightarrow> convex t \<Longrightarrow> convex (s \<inter> t)"
   unfolding convex_def by auto
 
+lemma convex_INT: "\<forall>i\<in>A. convex (B i) \<Longrightarrow> convex (\<Inter>i\<in>A. B i)"
+  unfolding convex_def by auto
+
+lemma convex_Times: "convex s \<Longrightarrow> convex t \<Longrightarrow> convex (s \<times> t)"
+  unfolding convex_def by auto
+
 lemma convex_halfspace_le: "convex {x. inner a x \<le> b}"
   unfolding convex_def
   by (auto simp: inner_add intro!: convex_bound_le)