src/HOLCF/ConvexPD.thy
changeset 33808 31169fdc5ae7
parent 33585 8d39394fe5cf
child 34973 ae634fad947e
--- a/src/HOLCF/ConvexPD.thy	Thu Nov 19 21:06:22 2009 -0800
+++ b/src/HOLCF/ConvexPD.thy	Thu Nov 19 21:44:37 2009 -0800
@@ -495,6 +495,9 @@
 lemma convex_map_ident: "convex_map\<cdot>(\<Lambda> x. x)\<cdot>xs = xs"
 by (induct xs rule: convex_pd_induct, simp_all)
 
+lemma convex_map_ID: "convex_map\<cdot>ID = ID"
+by (simp add: expand_cfun_eq ID_def convex_map_ident)
+
 lemma convex_map_map:
   "convex_map\<cdot>f\<cdot>(convex_map\<cdot>g\<cdot>xs) = convex_map\<cdot>(\<Lambda> x. f\<cdot>(g\<cdot>x))\<cdot>xs"
 by (induct xs rule: convex_pd_induct, simp_all)