src/Doc/Tutorial/Rules/find2.thy
changeset 69505 cc2d676d5395
parent 67406 23307fd33906
equal deleted inserted replaced
69504:bda7527ccf05 69505:cc2d676d5395
    11 For this purpose, \pgmenu{Find} provides three aditional search criteria:
    11 For this purpose, \pgmenu{Find} provides three aditional search criteria:
    12 \texttt{intro}, \texttt{elim} and \texttt{dest}.
    12 \texttt{intro}, \texttt{elim} and \texttt{dest}.
    13 
    13 
    14 For example, given the goal @{subgoals[display,indent=0,margin=65]}
    14 For example, given the goal @{subgoals[display,indent=0,margin=65]}
    15 you can click on \pgmenu{Find} and type in the search expression
    15 you can click on \pgmenu{Find} and type in the search expression
    16 \texttt{intro}. You will be shown a few rules ending in @{text"\<Longrightarrow> ?P \<and> ?Q"},
    16 \texttt{intro}. You will be shown a few rules ending in \<open>\<Longrightarrow> ?P \<and> ?Q\<close>,
    17 among them @{thm[source]conjI}\@. You may even discover that
    17 among them @{thm[source]conjI}\@. You may even discover that
    18 the very theorem you are trying to prove is already in the
    18 the very theorem you are trying to prove is already in the
    19 database.  Given the goal\<close>
    19 database.  Given the goal\<close>
    20 (*<*)
    20 (*<*)
    21 oops
    21 oops
    29 As before, search criteria can be combined freely: for example,
    29 As before, search criteria can be combined freely: for example,
    30 \begin{ttbox}
    30 \begin{ttbox}
    31 "_ \at\ _"  intro
    31 "_ \at\ _"  intro
    32 \end{ttbox}
    32 \end{ttbox}
    33 searches for all introduction rules that match the current goal and
    33 searches for all introduction rules that match the current goal and
    34 mention the @{text"@"} function.
    34 mention the \<open>@\<close> function.
    35 
    35 
    36 Searching for elimination and destruction rules via \texttt{elim} and
    36 Searching for elimination and destruction rules via \texttt{elim} and
    37 \texttt{dest} is analogous to \texttt{intro} but takes the assumptions
    37 \texttt{dest} is analogous to \texttt{intro} but takes the assumptions
    38 into account, too.
    38 into account, too.
    39 \<close>
    39 \<close>