src/Doc/Datatypes/Datatypes.thy
changeset 62747 f65ef4723aca
parent 62740 69e4a4fffea9
child 62756 d4b7d128ec5a
--- a/src/Doc/Datatypes/Datatypes.thy	Tue Mar 29 19:17:05 2016 +0200
+++ b/src/Doc/Datatypes/Datatypes.thy	Tue Mar 29 21:25:19 2016 +0200
@@ -3094,8 +3094,9 @@
 
 The syntactic entity \synt{target} can be used to specify a local context,
 \synt{name} denotes an identifier, \synt{typefree} denotes fixed type variable
-(@{typ 'a}, @{typ 'b}, \ldots), and \synt{mixfix} denotes the usual
-parenthesized mixfix notation @{cite "isabelle-isar-ref"}.
+(@{typ 'a}, @{typ 'b}, \ldots), \synt{mixfix} denotes the usual parenthesized
+mixfix notation, and \synt{types} denotes a space-separated list of types
+@{cite "isabelle-isar-ref"}.
 
 The @{syntax plugins} option indicates which plugins should be enabled
 (@{text only}) or disabled (@{text del}). By default, all plugins are enabled.