src/HOL/List.thy
changeset 35208 2b9bce05e84b
parent 35195 5163c2d00904
child 35217 01e968432467
--- a/src/HOL/List.thy	Thu Feb 18 08:17:24 2010 +0100
+++ b/src/HOL/List.thy	Thu Feb 18 16:08:26 2010 +0100
@@ -720,6 +720,11 @@
 lemma map_map [simp]: "map f (map g xs) = map (f \<circ> g) xs"
 by (induct xs) auto
 
+lemma map_comp_map[simp]: "((map f) o (map g)) = map(f o g)"
+apply(rule ext)
+apply(simp)
+done
+
 lemma rev_map: "rev (map f xs) = map f (rev xs)"
 by (induct xs) auto