src/HOL/IMP/Procs.thy
changeset 47818 151d137f1095
parent 45212 e87feee00a4c
child 51019 146f63c3f024
--- a/src/HOL/IMP/Procs.thy	Fri Apr 27 23:17:58 2012 +0200
+++ b/src/HOL/IMP/Procs.thy	Sat Apr 28 07:38:22 2012 +0200
@@ -9,7 +9,7 @@
 datatype
   com = SKIP 
       | Assign vname aexp        ("_ ::= _" [1000, 61] 61)
-      | Semi   com  com          ("_;/ _"  [60, 61] 60)
+      | Seq    com  com          ("_;/ _"  [60, 61] 60)
       | If     bexp com com     ("(IF _/ THEN _/ ELSE _)"  [0, 0, 61] 61)
       | While  bexp com         ("(WHILE _/ DO _)"  [0, 61] 61)
       | Var    vname com        ("(1{VAR _;;/ _})")