src/HOL/TLA/Stfun.thy
changeset 35108 e384e27c229f
parent 21624 6f79647cf536
child 35318 e1b61c5fd494
--- a/src/HOL/TLA/Stfun.thy	Thu Feb 11 13:54:53 2010 +0100
+++ b/src/HOL/TLA/Stfun.thy	Thu Feb 11 21:31:50 2010 +0100
@@ -1,8 +1,6 @@
-(*
-    File:        TLA/Stfun.thy
-    ID:          $Id$
-    Author:      Stephan Merz
-    Copyright:   1998 University of Munich
+(*  Title:      HOL/TLA/Stfun.thy
+    Author:     Stephan Merz
+    Copyright:  1998 University of Munich
 *)
 
 header {* States and state functions for TLA as an "intensional" logic *}
@@ -42,7 +40,7 @@
 
 translations
   "PRED P"   =>  "(P::state => _)"
-  "_stvars"  ==  "stvars"
+  "_stvars"  ==  "CONST stvars"
 
 defs
   (* Base variables may be assigned arbitrary (type-correct) values.