src/HOL/Record.thy
changeset 35146 f7bf73b0d7e5
parent 35145 f132a4fd8679
child 36176 3fe7e97ccca8
--- a/src/HOL/Record.thy	Tue Feb 16 14:08:39 2010 +0100
+++ b/src/HOL/Record.thy	Tue Feb 16 16:03:06 2010 +0100
@@ -420,7 +420,7 @@
 subsection {* Concrete record syntax *}
 
 nonterminals
-  ident field_type field_types field fields update updates
+  ident field_type field_types field fields field_update field_updates
 syntax
   "_constify"           :: "id => ident"                        ("_")
   "_constify"           :: "longid => ident"                    ("_")
@@ -437,17 +437,17 @@
   "_record"             :: "fields => 'a"                       ("(3'(| _ |'))")
   "_record_scheme"      :: "fields => 'a => 'a"                 ("(3'(| _,/ (2... =/ _) |'))")
 
-  "_update"             :: "ident => 'a => update"              ("(2_ :=/ _)")
-  ""                    :: "update => updates"                  ("_")
-  "_updates"            :: "update => updates => updates"       ("_,/ _")
-  "_record_update"      :: "'a => updates => 'b"                ("_/(3'(| _ |'))" [900, 0] 900)
+  "_field_update"       :: "ident => 'a => field_update"        ("(2_ :=/ _)")
+  ""                    :: "field_update => field_updates"      ("_")
+  "_field_updates"      :: "field_update => field_updates => field_updates"  ("_,/ _")
+  "_record_update"      :: "'a => field_updates => 'b"          ("_/(3'(| _ |'))" [900, 0] 900)
 
 syntax (xsymbols)
   "_record_type"        :: "field_types => type"                ("(3\<lparr>_\<rparr>)")
   "_record_type_scheme" :: "field_types => type => type"        ("(3\<lparr>_,/ (2\<dots> ::/ _)\<rparr>)")
   "_record"             :: "fields => 'a"                       ("(3\<lparr>_\<rparr>)")
   "_record_scheme"      :: "fields => 'a => 'a"                 ("(3\<lparr>_,/ (2\<dots> =/ _)\<rparr>)")
-  "_record_update"      :: "'a => updates => 'b"                ("_/(3\<lparr>_\<rparr>)" [900, 0] 900)
+  "_record_update"      :: "'a => field_updates => 'b"          ("_/(3\<lparr>_\<rparr>)" [900, 0] 900)
 
 
 subsection {* Record package *}