src/HOL/List.thy
changeset 23983 79dc793bec43
parent 23971 e6d505d5b03d
child 24037 0a41d2ebc0cd
--- a/src/HOL/List.thy	Wed Jul 25 17:05:50 2007 +0200
+++ b/src/HOL/List.thy	Wed Jul 25 18:10:28 2007 +0200
@@ -983,6 +983,9 @@
 lemma set_concat [simp]: "set (concat xs) = \<Union>(set ` set xs)"
 by (induct xs) auto
 
+lemma set_concat_map: "set(concat(map f xs)) = (UN x:set xs. set(f x))"
+by(auto)
+
 lemma map_concat: "map f (concat xs) = concat (map (map f) xs)"
 by (induct xs) auto
 
@@ -1556,6 +1559,10 @@
   "(x,y)\<in> set (zip xs ys) \<Longrightarrow> y \<in> set ys"
 by (induct xs ys rule:list_induct2') auto
 
+lemma in_set_zipE:
+  "(x,y) : set(zip xs ys) \<Longrightarrow> (\<lbrakk> x : set xs; y : set ys \<rbrakk> \<Longrightarrow> R) \<Longrightarrow> R"
+by(blast dest: set_zip_leftD set_zip_rightD)
+
 subsubsection {* @{text list_all2} *}
 
 lemma list_all2_lengthD [intro?]: