src/HOL/HoareParallel/OG_Tran.thy
changeset 30304 d8e4cd2ac2a1
parent 23746 a455e69c31cc
child 30952 7ab2716dd93b
--- a/src/HOL/HoareParallel/OG_Tran.thy	Thu Mar 05 08:23:10 2009 +0100
+++ b/src/HOL/HoareParallel/OG_Tran.thy	Thu Mar 05 08:23:11 2009 +0100
@@ -102,7 +102,7 @@
   "SEM c S \<equiv> \<Union>sem c ` S "
 
 syntax "_Omega" :: "'a com"    ("\<Omega>" 63)
-translations  "\<Omega>" \<rightleftharpoons> "While UNIV UNIV (Basic id)"
+translations  "\<Omega>" \<rightleftharpoons> "While CONST UNIV CONST UNIV (Basic id)"
 
 consts fwhile :: "'a bexp \<Rightarrow> 'a com \<Rightarrow> nat \<Rightarrow> 'a com"
 primrec