doc-src/ProgProve/Thys/Logic.thy
changeset 47727 027c7f8cef22
parent 47720 b11dac707c78
--- a/doc-src/ProgProve/Thys/Logic.thy	Tue Apr 24 11:07:50 2012 +0200
+++ b/doc-src/ProgProve/Thys/Logic.thy	Tue Apr 24 12:36:27 2012 +0200
@@ -244,6 +244,19 @@
 but we will not enlarge on that here.
 
 
+\subsubsection{Trying them all}
+
+If you want to try all of the above automatic proof methods you simply type
+\begin{isabelle}
+\isacom{try}
+\end{isabelle}
+You can also add specific simplification and introduction rules:
+\begin{isabelle}
+\isacom{try} @{text"simp: \<dots> intro: \<dots>"}
+\end{isabelle}
+There is also a lightweight variant \isacom{try0} that does not call
+sledgehammer.
+
 \subsection{Single step proofs}
 
 Although automation is nice, it often fails, at least initially, and you need
@@ -410,11 +423,19 @@
 text{* In this particular example we could have backchained with
 @{thm[source] Suc_leD}, too, but because the premise is more complicated than the conclusion this can easily lead to nontermination.
 
+\subsubsection{Finding theorems}
+
+Command \isacom{find\_theorems} searches for specific theorems in the current
+theory. Search criteria include pattern matching on terms and on names.
+For details see the Isabelle/Isar Reference Manual~\cite{IsarRef}.
+\bigskip
+
 \begin{warn}
 To ease readability we will drop the question marks
 in front of unknowns from now on.
 \end{warn}
 
+
 \section{Inductive definitions}
 \label{sec:inductive-defs}