src/HOL/Bali/State.thy
changeset 31127 b63c3f6bd3be
parent 30235 58d147683393
child 32960 69916a850301
--- a/src/HOL/Bali/State.thy	Tue May 12 20:07:05 2009 +0200
+++ b/src/HOL/Bali/State.thy	Tue May 12 21:17:34 2009 +0200
@@ -29,7 +29,7 @@
 types	vn   = "fspec + int"                    --{* variable name      *}
 record	obj  = 
           tag :: "obj_tag"                      --{* generalized object *}
-          values :: "(vn, val) table"      
+          "values" :: "(vn, val) table"      
 
 translations 
   "fspec" <= (type) "vname \<times> qtname"