src/HOL/Record.thy
changeset 10331 7411e4659d4a
parent 10309 a7f961fb62c6
child 10641 d1533f63c738
--- a/src/HOL/Record.thy	Wed Oct 25 18:31:21 2000 +0200
+++ b/src/HOL/Record.thy	Wed Oct 25 18:32:02 2000 +0200
@@ -40,7 +40,7 @@
   "_updates"            :: "[update, updates] => updates"               ("_,/ _")
   "_record_update"      :: "['a, updates] => 'b"                ("_/(3'(| _ |'))" [900,0] 900)
 
-syntax (input)   (* FIXME (xsymbols) *)
+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>)")