doc-src/IsarRef/Thy/Inner_Syntax.thy
changeset 28767 f09ceb800d00
parent 28766 accab7594b8e
child 28769 8fc228f21861
--- a/doc-src/IsarRef/Thy/Inner_Syntax.thy	Thu Nov 13 21:52:09 2008 +0100
+++ b/doc-src/IsarRef/Thy/Inner_Syntax.thy	Thu Nov 13 21:52:59 2008 +0100
@@ -246,11 +246,11 @@
 section {* Mixfix annotations *}
 
 text {* Mixfix annotations specify concrete \emph{inner syntax} of
-  Isabelle types and terms.  Some commands such as @{command "types"}
-  (see \secref{sec:types-pure}) admit infixes only, while @{command
-  "consts"} (see \secref{sec:consts}) and @{command "syntax"} (see
-  \secref{sec:syn-trans}) support the full range of general mixfixes
-  and binders.
+  Isabelle types and terms.  Some commands such as @{command
+  "typedecl"} admit infixes only, while @{command "definition"} etc.\
+  support the full range of general mixfixes and binders.  Fixed
+  parameters in toplevel theorem statements, locale specifications
+  also admit mixfix annotations.
 
   \indexouternonterm{infix}\indexouternonterm{mixfix}\indexouternonterm{structmixfix}
   \begin{rail}