src/ZF/UNITY/State.thy
changeset 14171 0cab06e3bbd0
parent 14084 ccb48f3239f7
child 16417 9bc16273c2d4
--- a/src/ZF/UNITY/State.thy	Wed Aug 27 18:22:34 2003 +0200
+++ b/src/ZF/UNITY/State.thy	Thu Aug 28 01:56:40 2003 +0200
@@ -23,7 +23,7 @@
 
 constdefs
   state   :: i
-   "state == \<Pi>x \<in> var. cons(default_val(x), type_of(x))"
+   "state == \<Pi> x \<in> var. cons(default_val(x), type_of(x))"
 
   st0     :: i
    "st0 == \<lambda>x \<in> var. default_val(x)"