src/HOLCF/Powerdomains.thy
changeset 35479 dffffe36344a
parent 35473 c4d3d65856dd
child 39973 c62b4ff97bfc
--- a/src/HOLCF/Powerdomains.thy	Sun Feb 28 18:12:08 2010 -0800
+++ b/src/HOLCF/Powerdomains.thy	Sun Feb 28 18:33:57 2010 -0800
@@ -298,13 +298,16 @@
 setup {*
   fold Domain_Isomorphism.add_type_constructor
     [(@{type_name "upper_pd"}, @{term upper_defl}, @{const_name upper_map},
-        @{thm REP_upper}, @{thm isodefl_upper}, @{thm upper_map_ID}),
+        @{thm REP_upper}, @{thm isodefl_upper}, @{thm upper_map_ID},
+          @{thm deflation_upper_map}),
 
      (@{type_name "lower_pd"}, @{term lower_defl}, @{const_name lower_map},
-        @{thm REP_lower}, @{thm isodefl_lower}, @{thm lower_map_ID}),
+        @{thm REP_lower}, @{thm isodefl_lower}, @{thm lower_map_ID},
+          @{thm deflation_lower_map}),
 
      (@{type_name "convex_pd"}, @{term convex_defl}, @{const_name convex_map},
-        @{thm REP_convex}, @{thm isodefl_convex}, @{thm convex_map_ID})]
+        @{thm REP_convex}, @{thm isodefl_convex}, @{thm convex_map_ID},
+          @{thm deflation_convex_map})]
 *}
 
 end