added bulkload
authorhaftmann
Sat, 07 Feb 2009 09:57:03 +0100
changeset 29828 2bc09b164f2b
parent 29827 c82b3e8a4daf
child 29829 9acb915a62fa
added bulkload
src/HOL/Library/Mapping.thy
--- a/src/HOL/Library/Mapping.thy	Sat Feb 07 08:37:43 2009 +0100
+++ b/src/HOL/Library/Mapping.thy	Sat Feb 07 09:57:03 2009 +0100
@@ -127,14 +127,6 @@
   "size (tabulate ks f) = length (remdups ks)"
   by (simp add: size_def keys_tabulate distinct_card [of "remdups ks", symmetric])
 
-lemma zip_map_fst_snd: (*FIXME move*)
-  "zip (map fst zs) (map snd zs) = zs"
-  by (induct zs) simp_all
-
-lemma zip_eq_conv: (*FIXME move*)
-  "length xs = length ys \<Longrightarrow> zip xs ys = zs \<longleftrightarrow> map fst zs = xs \<and> map snd zs = ys"
-  by (auto simp add: zip_map_fst_snd)
-
 lemma bulkload_tabulate: (*FIXME Isar proof*)
   "bulkload xs = tabulate [0..<length xs] (nth xs)"
   unfolding bulkload_def tabulate_def apply simp