src/HOLCF/Powerdomains.thy
changeset 40218 f7d4d023a899
parent 40216 366309dfaf60
child 40487 1320a0747974
--- a/src/HOLCF/Powerdomains.thy	Wed Oct 27 11:06:53 2010 -0700
+++ b/src/HOLCF/Powerdomains.thy	Wed Oct 27 11:10:36 2010 -0700
@@ -43,9 +43,9 @@
 
 setup {*
   fold Domain_Isomorphism.add_type_constructor
-    [(@{type_name "upper_pd"}, @{term upper_defl}, @{const_name upper_map}),
-     (@{type_name "lower_pd"}, @{term lower_defl}, @{const_name lower_map}),
-     (@{type_name "convex_pd"}, @{term convex_defl}, @{const_name convex_map})]
+    [(@{type_name "upper_pd"}, @{const_name upper_defl}, @{const_name upper_map}, [true]),
+     (@{type_name "lower_pd"}, @{const_name lower_defl}, @{const_name lower_map}, [true]),
+     (@{type_name "convex_pd"}, @{const_name convex_defl}, @{const_name convex_map}, [true])]
 *}
 
 end