aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
authorGravatar puech <puech@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-03-11 15:42:31 +0000
committerGravatar puech <puech@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-03-11 15:42:31 +0000
commit8a944fd93df07453cba53b752670ae451c370a65 (patch)
treef28239891bc5bcd7f0e309247fcfad23fa394885
parentb75171fe23f0a0d691961444100710e73e34aa92 (diff)
Update manual on search commands
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12861 85f007b7-540e-0410-9357-904b9bb8a0f7
-rw-r--r--doc/refman/RefMan-oth.tex31
1 files changed, 17 insertions, 14 deletions
diff --git a/doc/refman/RefMan-oth.tex b/doc/refman/RefMan-oth.tex
index c71df4e22..9e18d0af2 100644
--- a/doc/refman/RefMan-oth.tex
+++ b/doc/refman/RefMan-oth.tex
@@ -99,25 +99,25 @@ relies.
to the assumptions.
\end{Variants}
-\subsection[\tt Search {\qualid}.]{\tt Search {\qualid}.\comindex{Search}}
+\subsection[\tt Search {\term}.]{\tt Search {\term}.\comindex{Search}}
This command displays the name and type of all theorems of the current
-context whose statement's conclusion has the form {\tt ({\qualid} t1 ..
+context whose statement's conclusion has the form {\tt ({\term} t1 ..
tn)}. This command is useful to remind the user of the name of
library lemmas.
-\begin{ErrMsgs}
-\item \errindex{The reference \qualid\ was not found in the current
-environment}\\
- There is no constant in the environment named \qualid.
-\end{ErrMsgs}
+
+\begin{coq_example}
+Search le.
+Search (@eq bool).
+\end{coq_example}
\begin{Variants}
\item
-{\tt Search {\qualid} inside {\module$_1$} \ldots{} {\module$_n$}.}
+{\tt Search {\term} inside {\module$_1$} \ldots{} {\module$_n$}.}
This restricts the search to constructions defined in modules
{\module$_1$} \ldots{} {\module$_n$}.
-\item {\tt Search {\qualid} outside {\module$_1$} \ldots{} {\module$_n$}.}
+\item {\tt Search {\term} outside {\module$_1$} \ldots{} {\module$_n$}.}
This restricts the search to constructions not defined in modules
{\module$_1$} \ldots{} {\module$_n$}.
@@ -218,15 +218,18 @@ SearchAbout (?x * _ + ?x * _)%Z outside OmegaLemmas.
\subsection[\tt SearchPattern {\termpattern}.]{\tt SearchPattern {\term}.\comindex{SearchPattern}}
This command displays the name and type of all theorems of the current
-context whose statement's conclusion matches the expression {\term}
-where holes in the latter are denoted by ``{\texttt \_}''. It is a
-variant of {\tt SearchAbout {\termpattern}} that does not look for
-subterms but searches for statements whose conclusion has exactly the
-expected form.
+context whose statement's conclusion or last hypothesis and conclusion
+matches the expression {\term} where holes in the latter are denoted
+by ``{\texttt \_}''. It is a variant of {\tt SearchAbout
+ {\termpattern}} that does not look for subterms but searches for
+statements whose conclusion has exactly the expected form, or whose
+statement finishes by the given series of hypothesis/conclusion.
\begin{coq_example}
Require Import Arith.
SearchPattern (_ + _ = _ + _).
+SearchPattern (nat -> bool).
+SearchPattern (forall l : list _, _ l l).
\end{coq_example}
Patterns need not be linear: you can express that the same expression