doc-src/IsarRef/Thy/Proof.thy
changeset 42705 528a2ba8fa74
parent 42704 3f19e324ff59
child 42813 6c841fa92fa2
--- a/doc-src/IsarRef/Thy/Proof.thy	Thu May 05 23:15:11 2011 +0200
+++ b/doc-src/IsarRef/Thy/Proof.thy	Thu May 05 23:23:02 2011 +0200
@@ -194,7 +194,7 @@
     ;
     @@{command def} (def + @'and')
     ;
-    def: @{syntax thmdecl}? \\ @{syntax name} ('==' | '\<equiv>') @{syntax term} @{syntax termpat}?
+    def: @{syntax thmdecl}? \\ @{syntax name} ('==' | '\<equiv>') @{syntax term} @{syntax term_pat}?
   "}
 
   \begin{description}
@@ -269,8 +269,8 @@
     @@{command let} ((@{syntax term} + @'and') '=' @{syntax term} + @'and')
   "}
 
-  The syntax of @{keyword "is"} patterns follows @{syntax termpat} or
-  @{syntax proppat} (see \secref{sec:term-decls}).
+  The syntax of @{keyword "is"} patterns follows @{syntax term_pat} or
+  @{syntax prop_pat} (see \secref{sec:term-decls}).
 
   \begin{description}
 
@@ -568,7 +568,7 @@
   "n"}.
 
   @{rail "
-    @{syntax_def goalspec}:
+    @{syntax_def goal_spec}:
       '[' (@{syntax nat} '-' @{syntax nat} | @{syntax nat} '-' | @{syntax nat} | '!' ) ']'
   "}
 *}