src/Doc/Isar_Ref/Misc.thy
changeset 59917 9830c944670f
parent 58618 782f0b662cae
child 60270 a147272b16f9
--- a/src/Doc/Isar_Ref/Misc.thy	Fri Apr 03 18:36:19 2015 +0200
+++ b/src/Doc/Isar_Ref/Misc.thy	Fri Apr 03 19:56:51 2015 +0200
@@ -21,9 +21,12 @@
   \end{matharray}
 
   @{rail \<open>
-    (@@{command print_theory} | @@{command print_theorems} | @@{command print_facts}) ('!'?)
+    (@@{command print_theory} |
+      @@{command print_methods} |
+      @@{command print_attributes} |
+      @@{command print_theorems} |
+      @@{command print_facts}) ('!'?)
     ;
-
     @@{command find_theorems} ('(' @{syntax nat}? 'with_dups'? ')')? \<newline> (thmcriterion * )
     ;
     thmcriterion: ('-'?) ('name' ':' @{syntax nameref} | 'intro' | 'elim' | 'dest' |
@@ -45,23 +48,24 @@
 
   \begin{description}
   
-  \item @{command "print_theory"} prints the main logical content of
-  the background theory; the ``@{text "!"}'' option indicates extra
+  \item @{command "print_theory"} prints the main logical content of the
+  background theory; the ``@{text "!"}'' option indicates extra verbosity.
+
+  \item @{command "print_methods"} prints all proof methods available in the
+  current theory context; the ``@{text "!"}'' option indicates extra
   verbosity.
-
-  \item @{command "print_methods"} prints all proof methods
-  available in the current theory context.
   
-  \item @{command "print_attributes"} prints all attributes
-  available in the current theory context.
+  \item @{command "print_attributes"} prints all attributes available in the
+  current theory context; the ``@{text "!"}'' option indicates extra
+  verbosity.
   
-  \item @{command "print_theorems"} prints theorems of the background
-  theory resulting from the last command; the ``@{text "!"}'' option
-  indicates extra verbosity.
+  \item @{command "print_theorems"} prints theorems of the background theory
+  resulting from the last command; the ``@{text "!"}'' option indicates
+  extra verbosity.
   
-  \item @{command "print_facts"} prints all local facts of the
-  current context, both named and unnamed ones; the ``@{text "!"}''
-  option indicates extra verbosity.
+  \item @{command "print_facts"} prints all local facts of the current
+  context, both named and unnamed ones; the ``@{text "!"}'' option indicates
+  extra verbosity.
   
   \item @{command "print_term_bindings"} prints all term bindings that
   are present in the context.