src/HOL/Map.thy
changeset 33635 dcaada178c6f
parent 32236 0203e1006f1b
child 34941 156925dd67af
--- a/src/HOL/Map.thy	Wed Nov 11 21:53:58 2009 +0100
+++ b/src/HOL/Map.thy	Thu Nov 12 15:10:24 2009 +0100
@@ -218,6 +218,10 @@
   ultimately show ?case by simp
 qed
 
+lemma map_of_zip_map:
+  "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 finite_range_map_of: "finite (range (map_of xys))"
 apply (induct xys)
  apply (simp_all add: image_constant)