src/HOL/Bali/Basis.thy
changeset 33965 f57c11db4ad4
parent 32960 69916a850301
child 34915 7894c7dab132
--- a/src/HOL/Bali/Basis.thy	Fri Nov 27 08:42:34 2009 +0100
+++ b/src/HOL/Bali/Basis.thy	Fri Nov 27 08:42:50 2009 +0100
@@ -216,8 +216,8 @@
          In1l   :: "'al \<Rightarrow> ('al + 'ar, 'b, 'c) sum3"
          In1r   :: "'ar \<Rightarrow> ('al + 'ar, 'b, 'c) sum3"
 translations
-        "In1l e" == "In1 (Inl e)"
-        "In1r c" == "In1 (Inr c)"
+        "In1l e" == "In1 (CONST Inl e)"
+        "In1r c" == "In1 (CONST Inr c)"
 
 syntax the_In1l :: "('al + 'ar, 'b, 'c) sum3 \<Rightarrow> 'al"
        the_In1r :: "('al + 'ar, 'b, 'c) sum3 \<Rightarrow> 'ar"
@@ -233,7 +233,7 @@
 (* e.g. lemmas is_stmt_rews = is_stmt_def [of "In1l x", simplified] *)
 
 translations
-  "option"<= (type) "Datatype.option"
+  "option"<= (type) "Option.option"
   "list"  <= (type) "List.list"
   "sum3"  <= (type) "Basis.sum3"