diff -r 90cd3c53a887 -r bc01725d7918 src/HOL/IMP/Abs_Int_ITP/Abs_Int1_ITP.thy --- 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 \ None | Some S \ 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 \ post c2})" |