src/HOLCF/Representable.thy
changeset 33809 033831fd9ef3
parent 33794 364bc92ba081
child 35431 8758fe1fc9f8
child 35473 c4d3d65856dd
--- a/src/HOLCF/Representable.thy	Thu Nov 19 21:44:37 2009 -0800
+++ b/src/HOLCF/Representable.thy	Thu Nov 19 22:25:11 2009 -0800
@@ -1038,28 +1038,28 @@
 setup {*
   fold Domain_Isomorphism.add_type_constructor
     [(@{type_name "->"}, @{term cfun_defl}, @{const_name cfun_map},
-        @{thm REP_cfun}, @{thm isodefl_cfun}),
+        @{thm REP_cfun}, @{thm isodefl_cfun}, @{thm cfun_map_ID}),
 
      (@{type_name "++"}, @{term ssum_defl}, @{const_name ssum_map},
-        @{thm REP_ssum}, @{thm isodefl_ssum}),
+        @{thm REP_ssum}, @{thm isodefl_ssum}, @{thm ssum_map_ID}),
 
      (@{type_name "**"}, @{term sprod_defl}, @{const_name sprod_map},
-        @{thm REP_sprod}, @{thm isodefl_sprod}),
+        @{thm REP_sprod}, @{thm isodefl_sprod}, @{thm sprod_map_ID}),
 
      (@{type_name "*"}, @{term cprod_defl}, @{const_name cprod_map},
-        @{thm REP_cprod}, @{thm isodefl_cprod}),
+        @{thm REP_cprod}, @{thm isodefl_cprod}, @{thm cprod_map_ID}),
 
      (@{type_name "u"}, @{term u_defl}, @{const_name u_map},
-        @{thm REP_up}, @{thm isodefl_u}),
+        @{thm REP_up}, @{thm isodefl_u}, @{thm u_map_ID}),
 
      (@{type_name "upper_pd"}, @{term upper_defl}, @{const_name upper_map},
-        @{thm REP_upper}, @{thm isodefl_upper}),
+        @{thm REP_upper}, @{thm isodefl_upper}, @{thm upper_map_ID}),
 
      (@{type_name "lower_pd"}, @{term lower_defl}, @{const_name lower_map},
-        @{thm REP_lower}, @{thm isodefl_lower}),
+        @{thm REP_lower}, @{thm isodefl_lower}, @{thm lower_map_ID}),
 
      (@{type_name "convex_pd"}, @{term convex_defl}, @{const_name convex_map},
-        @{thm REP_convex}, @{thm isodefl_convex})]
+        @{thm REP_convex}, @{thm isodefl_convex}, @{thm convex_map_ID})]
 *}
 
 end