doc-src/TutorialI/Misc/simp.thy
changeset 16544 29828ddbf6ee
parent 16523 f8a734dc0fbc
child 16560 bed540afd4b3
equal deleted inserted replaced
16543:4dd8b4d1cfc3 16544:29828ddbf6ee
   416 
   416 
   417 In more complicated cases, the trace can be very lengthy.  Thus it is
   417 In more complicated cases, the trace can be very lengthy.  Thus it is
   418 advisable to reset the \pgmenu{Trace Simplifier} flag after having
   418 advisable to reset the \pgmenu{Trace Simplifier} flag after having
   419 obtained the desired trace.  *}
   419 obtained the desired trace.  *}
   420 
   420 
   421 subsection{*Finding Theorems*}
   421 subsection{*Finding Theorems\label{sec:find}*}
   422 
   422 
   423 text{*\indexbold{finding theorems}\indexbold{searching theorems}
   423 text{*\indexbold{finding theorems}\indexbold{searching theorems}
   424 Isabelle's large database of already proved theorems requires
   424 Isabelle's large database of already proved theorems requires
   425 and offers a powerful yet simple search engine. Its only limitation is
   425 and offers a powerful yet simple search engine. Its only limitation is
   426 its restriction to the theories currently loaded.
   426 its restriction to the theories currently loaded.
   492 "_ + _"  -"_ - _"  -simp: "_ * (_ + _)"  name: assoc
   492 "_ + _"  -"_ - _"  -simp: "_ * (_ + _)"  name: assoc
   493 \end{ttbox}
   493 \end{ttbox}
   494 looks for theorems containg a plus but no minus which do not simplify
   494 looks for theorems containg a plus but no minus which do not simplify
   495 \mbox{@{text"_ * (_ + _)"}} at the root and whose name contains \texttt{assoc}.
   495 \mbox{@{text"_ * (_ + _)"}} at the root and whose name contains \texttt{assoc}.
   496 
   496 
   497 Further search criteria are explained in \S\ref{sec:find:ied}.
   497 Further search criteria are explained in \S\ref{sec:find2}.
   498 
   498 
   499 \begin{pgnote}
   499 \begin{pgnote}
   500 Proof General keeps a history of all your search expressions.
   500 Proof General keeps a history of all your search expressions.
   501 If you click on \pgmenu{Find}, you can use the arrow keys to scroll
   501 If you click on \pgmenu{Find}, you can use the arrow keys to scroll
   502 through previous searches and just modify them. This saves you having
   502 through previous searches and just modify them. This saves you having