src/HOL/Bali/AxSem.thy
changeset 24783 5a3e336a2e37
parent 24038 18182c4aec9e
child 26342 0f65fa163304
--- a/src/HOL/Bali/AxSem.thy	Sun Sep 30 16:53:08 2007 +0200
+++ b/src/HOL/Bali/AxSem.thy	Sun Sep 30 21:55:15 2007 +0200
@@ -49,9 +49,9 @@
   "Vals x"     => "(In3 x)"
 
 syntax
-  "Val_"    :: "[pttrn] => pttrn"     ("Val:_"  [951] 950)
-  "Var_"    :: "[pttrn] => pttrn"     ("Var:_"  [951] 950)
-  "Vals_"   :: "[pttrn] => pttrn"     ("Vals:_" [951] 950)
+  "_Val"    :: "[pttrn] => pttrn"     ("Val:_"  [951] 950)
+  "_Var"    :: "[pttrn] => pttrn"     ("Var:_"  [951] 950)
+  "_Vals"   :: "[pttrn] => pttrn"     ("Vals:_" [951] 950)
 
 translations
   "\<lambda>Val:v . b"  == "(\<lambda>v. b) \<circ> the_In1"