src/HOL/TLA/Stfun.thy
changeset 35354 2e8dc3c64430
parent 35318 e1b61c5fd494
child 42018 878f33040280
--- a/src/HOL/TLA/Stfun.thy	Wed Feb 24 21:59:21 2010 +0100
+++ b/src/HOL/TLA/Stfun.thy	Wed Feb 24 22:04:10 2010 +0100
@@ -35,7 +35,7 @@
   stvars    :: "'a stfun => bool"
 
 syntax
-  "PRED"    :: "lift => 'a"                          ("PRED _")
+  "_PRED"   :: "lift => 'a"                          ("PRED _")
   "_stvars" :: "lift => bool"                        ("basevars _")
 
 translations