generalized lemma map_of_zip_map
authorhaftmann
Mon, 18 May 2009 15:45:36 +0200
changeset 31193 f8d4ac84334f
parent 31192 a324d214009c
child 31194 1d6926f96440
generalized lemma map_of_zip_map
src/HOL/Library/Enum.thy
--- a/src/HOL/Library/Enum.thy	Mon May 18 15:45:34 2009 +0200
+++ b/src/HOL/Library/Enum.thy	Mon May 18 15:45:36 2009 +0200
@@ -116,9 +116,8 @@
     by (simp add: length_n_lists)
 qed
 
-lemma map_of_zip_map:
-  fixes f :: "'a\<Colon>enum \<Rightarrow> 'b\<Colon>enum"
-  shows "map_of (zip xs (map f xs)) = (\<lambda>x. if x \<in> set xs then Some (f x) else None)"
+lemma map_of_zip_map: (*FIXME move to Map.thy*)
+  "map_of (zip xs (map f xs)) = (\<lambda>x. if x \<in> set xs then Some (f x) else None)"
   by (induct xs) (simp_all add: expand_fun_eq)
 
 lemma map_of_zip_enum_is_Some: