src/HOL/IMP/Collecting.thy
changeset 46070 8392c28d7868
parent 46069 4869f1389333
child 46116 b903d272c37d
--- a/src/HOL/IMP/Collecting.thy	Mon Jan 02 11:33:50 2012 +0100
+++ b/src/HOL/IMP/Collecting.thy	Mon Jan 02 11:54:21 2012 +0100
@@ -149,8 +149,8 @@
 "step S ({Inv} WHILE b DO c {P}) =
   {S \<union> post c} WHILE b DO (step {s:Inv. bval b s} c) {{s:Inv. \<not> bval b s}}"
 
-definition CS :: "state set \<Rightarrow> com \<Rightarrow> state set acom" where
-"CS S c = lfp (step S) c"
+definition CS :: "com \<Rightarrow> state set acom" where
+"CS c = lfp (step UNIV) c"
 
 lemma mono_step_aux: "x \<le> y \<Longrightarrow> S \<subseteq> T \<Longrightarrow> step S x \<le> step T y"
 proof(induction x y arbitrary: S T rule: less_eq_acom.induct)
@@ -174,10 +174,10 @@
 apply(simp add: strip_step)
 done
 
-lemma CS_unfold: "CS S c = step S (CS S c)"
+lemma CS_unfold: "CS c = step UNIV (CS c)"
 by (metis CS_def lfp_cs_unfold)
 
-lemma strip_CS[simp]: "strip(CS S c) = c"
+lemma strip_CS[simp]: "strip(CS c) = c"
 by(simp add: CS_def index_lfp[simplified])
 
 end