doc-src/IsarRef/Thy/Inner_Syntax.thy
changeset 41229 d797baa3d57c
parent 40879 ca132ef44944
child 42247 12fe41a92cd5
--- a/doc-src/IsarRef/Thy/Inner_Syntax.thy	Fri Dec 17 17:08:56 2010 +0100
+++ b/doc-src/IsarRef/Thy/Inner_Syntax.thy	Fri Dec 17 17:43:54 2010 +0100
@@ -723,7 +723,7 @@
 
 text {*
   \begin{matharray}{rcl}
-    @{command_def "nonterminals"} & : & @{text "theory \<rightarrow> theory"} \\
+    @{command_def "nonterminal"} & : & @{text "theory \<rightarrow> theory"} \\
     @{command_def "syntax"} & : & @{text "theory \<rightarrow> theory"} \\
     @{command_def "no_syntax"} & : & @{text "theory \<rightarrow> theory"} \\
     @{command_def "translations"} & : & @{text "theory \<rightarrow> theory"} \\
@@ -731,7 +731,7 @@
   \end{matharray}
 
   \begin{rail}
-    'nonterminals' (name +)
+    'nonterminal' (name + 'and')
     ;
     ('syntax' | 'no_syntax') mode? (constdecl +)
     ;
@@ -746,7 +746,7 @@
 
   \begin{description}
   
-  \item @{command "nonterminals"}~@{text c} declares a type
+  \item @{command "nonterminal"}~@{text c} declares a type
   constructor @{text c} (without arguments) to act as purely syntactic
   type: a nonterminal symbol of the inner syntax.