src/HOL/IMP/Abs_Int_ITP/Abs_Int1_ITP.thy
changeset 52046 bc01725d7918
parent 47818 151d137f1095
child 53015 a1119cf551e8
--- a/src/HOL/IMP/Abs_Int_ITP/Abs_Int1_ITP.thy	Fri May 17 02:57:00 2013 +0200
+++ b/src/HOL/IMP/Abs_Int_ITP/Abs_Int1_ITP.thy	Fri May 17 08:19:52 2013 +0200
@@ -33,7 +33,7 @@
 "step' S (SKIP {P}) = (SKIP {S})" |
 "step' S (x ::= e {P}) =
   x ::= e {case S of None \<Rightarrow> None | Some S \<Rightarrow> Some(update S x (aval' e S))}" |
-"step' S (c1; c2) = step' S c1; step' (post c1) c2" |
+"step' S (c1;; c2) = step' S c1;; step' (post c1) c2" |
 "step' S (IF b THEN c1 ELSE c2 {P}) =
   (let c1' = step' S c1; c2' = step' S c2
    in IF b THEN c1' ELSE c2' {post c1 \<squnion> post c2})" |