src/HOL/IMP/Denotation.thy
changeset 2847 6226b83ce2d8
parent 1696 e84bff5c519b
child 4897 be11be0b6ea1
--- a/src/HOL/IMP/Denotation.thy	Thu Mar 27 17:46:24 1997 +0100
+++ b/src/HOL/IMP/Denotation.thy	Sun Mar 30 13:40:38 1997 +0200
@@ -13,7 +13,7 @@
 constdefs
   Gamma :: [bexp,com_den] => (com_den => com_den)
            "Gamma b cd == (%phi.{(s,t). (s,t) : (phi O cd) & b(s)} Un 
-                                 {(s,t). (s,t) : id & ~b(s)})"
+                                 {(s,t). s=t & ~b(s)})"
     
 consts
   C     :: com => com_den