doc-src/IsarRef/Thy/HOL_Specific.thy
changeset 43040 665623e695ea
parent 43019 619f16bf2150
child 43270 bc72c1ccc89e
--- a/doc-src/IsarRef/Thy/HOL_Specific.thy	Fri May 27 10:33:16 2011 +0200
+++ b/doc-src/IsarRef/Thy/HOL_Specific.thy	Fri May 27 10:41:09 2011 +0200
@@ -931,15 +931,20 @@
 
   \begin{matharray}{rcl}
     @{command_def (HOL) "solve_direct"}@{text "\<^sup>*"} & : & @{text "proof \<rightarrow>"} \\
+    @{command_def (HOL) "try"}@{text "\<^sup>*"} & : & @{text "proof \<rightarrow>"} \\
     @{command_def (HOL) "try_methods"}@{text "\<^sup>*"} & : & @{text "proof \<rightarrow>"} \\
     @{command_def (HOL) "sledgehammer"}@{text "\<^sup>*"} & : & @{text "proof \<rightarrow>"} \\
     @{command_def (HOL) "sledgehammer_params"} & : & @{text "theory \<rightarrow> theory"}
   \end{matharray}
 
   @{rail "
+    @@{command (HOL) try}
+    ;
+
     @@{command (HOL) try_methods} ( ( ( 'simp' | 'intro' | 'elim' | 'dest' ) ':' @{syntax thmrefs} ) + ) ?
       @{syntax nat}?
     ;
+
     @@{command (HOL) sledgehammer} ( '[' args ']' )? facts? @{syntax nat}?
     ;