src/HOL/IMP/Abs_Int2.thy
changeset 46070 8392c28d7868
parent 46068 b9d4ec0f79ac
child 46153 7e4a18db7384
--- a/src/HOL/IMP/Abs_Int2.thy	Mon Jan 02 11:33:50 2012 +0100
+++ b/src/HOL/IMP/Abs_Int2.thy	Mon Jan 02 11:54:21 2012 +0100
@@ -187,7 +187,7 @@
 definition AI_WN :: "com \<Rightarrow> 'av st option acom option" where
 "AI_WN = pfp_WN (step' \<top>)"
 
-lemma AI_WN_sound: "AI_WN c = Some c' \<Longrightarrow> CS UNIV c \<le> \<gamma>\<^isub>c c'"
+lemma AI_WN_sound: "AI_WN c = Some c' \<Longrightarrow> CS c \<le> \<gamma>\<^isub>c c'"
 proof(simp add: CS_def AI_WN_def)
   assume 1: "pfp_WN (step' \<top>) c = Some c'"
   from pfp_WN_pfp[OF allI[OF strip_step'] mono_step' 1]