src/HOL/IMP/Abs_Int0.thy
changeset 46070 8392c28d7868
parent 46068 b9d4ec0f79ac
child 46153 7e4a18db7384
--- a/src/HOL/IMP/Abs_Int0.thy	Mon Jan 02 11:33:50 2012 +0100
+++ b/src/HOL/IMP/Abs_Int0.thy	Mon Jan 02 11:54:21 2012 +0100
@@ -91,7 +91,7 @@
   ultimately show ?case by (simp add: While.IH subset_iff)
 qed
 
-lemma AI_sound: "AI c = Some c' \<Longrightarrow> CS UNIV c \<le> \<gamma>\<^isub>c c'"
+lemma AI_sound: "AI c = Some c' \<Longrightarrow> CS c \<le> \<gamma>\<^isub>c c'"
 proof(simp add: CS_def AI_def)
   assume 1: "lpfp\<^isub>c (step' \<top>) c = Some c'"
   have 2: "step' \<top> c' \<sqsubseteq> c'" by(rule lpfpc_pfp[OF 1])