tuned
authornipkow
Thu, 27 Sep 2012 10:43:40 +0200
changeset 49604 c54d901d2946
parent 49603 a115dda10251
child 49605 ea566f5e1724
child 49615 e0e8b53534de
tuned
src/HOL/IMP/Collecting.thy
--- a/src/HOL/IMP/Collecting.thy	Thu Sep 27 10:20:38 2012 +0200
+++ b/src/HOL/IMP/Collecting.thy	Thu Sep 27 10:43:40 2012 +0200
@@ -144,11 +144,11 @@
 fun step :: "state set \<Rightarrow> state set acom \<Rightarrow> state set acom" where
 "step S (SKIP {P}) = (SKIP {S})" |
 "step S (x ::= e {P}) =
-  (x ::= e {{s'. EX s:S. s' = s(x := aval e s)}})" |
+  x ::= e {{s(x := aval e s) |s. s : S}}" |
 "step S (C1; C2) = step S C1; step (post C1) C2" |
 "step S (IF b THEN {P1} C1 ELSE {P2} C2 {P}) =
-   IF b THEN {{s:S. bval b s}} step P1 C1 ELSE {{s:S. \<not> bval b s}} step P2 C2
-   {post C1 \<union> post C2}" |
+  IF b THEN {{s:S. bval b s}} step P1 C1 ELSE {{s:S. \<not> bval b s}} step P2 C2
+  {post C1 \<union> post C2}" |
 "step S ({I} WHILE b DO {P} C {P'}) =
   {S \<union> post C} WHILE b DO {{s:I. bval b s}} step P C {{s:I. \<not> bval b s}}"