doc-src/IsarRef/Thy/Inner_Syntax.thy
changeset 39165 e790a5560834
parent 39137 ccb53edd59f0
child 39279 878d86983dc1
--- a/doc-src/IsarRef/Thy/Inner_Syntax.thy	Mon Sep 06 22:08:49 2010 +0200
+++ b/doc-src/IsarRef/Thy/Inner_Syntax.thy	Mon Sep 06 22:31:54 2010 +0200
@@ -33,7 +33,7 @@
     ;
     ( 'prf' | 'full\_prf' ) modes? thmrefs?
     ;
-    'pr' modes? nat? (',' nat)?
+    'pr' modes? nat?
     ;
 
     modes: '(' (name + ) ')'
@@ -69,11 +69,11 @@
   compact proof term, which is denoted by ``@{text _}'' placeholders
   there.
 
-  \item @{command "pr"}~@{text "goals, prems"} prints the current
-  proof state (if present), including the proof context, current facts
-  and goals.  The optional limit arguments affect the number of goals
-  and premises to be displayed, which is initially 10 for both.
-  Omitting limit values leaves the current setting unchanged.
+  \item @{command "pr"}~@{text "goals"} prints the current proof state
+  (if present), including current facts and goals.  The optional limit
+  arguments affect the number of goals to be displayed, which is
+  initially 10.  Omitting limit value leaves the current setting
+  unchanged.
 
   \end{description}