src/HOL/IMP/Com.thy
changeset 27362 a6dc1769fdda
parent 16417 9bc16273c2d4
child 41589 bbd861837ebc
--- a/src/HOL/IMP/Com.thy	Wed Jun 25 21:25:51 2008 +0200
+++ b/src/HOL/IMP/Com.thy	Wed Jun 25 22:01:34 2008 +0200
@@ -28,9 +28,9 @@
       | Cond   bexp com com     ("IF _ THEN _ ELSE _"  60)
       | While  bexp com         ("WHILE _ DO _"  60)
 
-syntax (latex)
-  SKIP :: com   ("\<SKIP>")
-  Cond :: "bexp \<Rightarrow> com \<Rightarrow> com \<Rightarrow> com"  ("\<IF> _ \<THEN> _ \<ELSE> _"  60)
-  While :: "bexp \<Rightarrow> com \<Rightarrow> com" ("\<WHILE> _ \<DO> _"  60)
+notation (latex)
+  SKIP  ("\<SKIP>") and
+  Cond  ("\<IF> _ \<THEN> _ \<ELSE> _"  60) and
+  While  ("\<WHILE> _ \<DO> _"  60)
 
 end