new lemmas
authorhuffman
Thu, 11 Jun 2009 08:26:08 -0700
changeset 31562 10d0fb526643
parent 31561 a5e168fd2bb9
child 31563 ded2364d14d4
new lemmas
src/HOL/Library/Product_Vector.thy
--- a/src/HOL/Library/Product_Vector.thy	Wed Jun 10 15:32:02 2009 -0700
+++ b/src/HOL/Library/Product_Vector.thy	Thu Jun 11 08:26:08 2009 -0700
@@ -72,6 +72,21 @@
 
 end
 
+lemma open_Times: "open S \<Longrightarrow> open T \<Longrightarrow> open (S \<times> T)"
+unfolding open_prod_def by auto
+
+lemma fst_vimage_eq_Times: "fst -` S = S \<times> UNIV"
+by auto
+
+lemma snd_vimage_eq_Times: "snd -` S = UNIV \<times> S"
+by auto
+
+lemma open_vimage_fst: "open S \<Longrightarrow> open (fst -` S)"
+by (simp add: fst_vimage_eq_Times open_Times)
+
+lemma open_vimage_snd: "open S \<Longrightarrow> open (snd -` S)"
+by (simp add: snd_vimage_eq_Times open_Times)
+
 subsection {* Product is a metric space *}
 
 instantiation