aboutsummaryrefslogtreecommitdiffhomepage
path: root/doc
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-05-20 08:45:22 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-05-20 08:45:22 +0000
commitfcb04fbe8d6b82aa02d266db6d200b9fcb6ace04 (patch)
tree8a7b87b64e7d03cbd8b83ed69956c78d5a095247 /doc
parent7590031325b144f6864d2194a700a92145617c13 (diff)
Ajout 'in (Type of ...)'
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@8334 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'doc')
-rw-r--r--doc/RefMan-tac.tex7
1 files changed, 4 insertions, 3 deletions
diff --git a/doc/RefMan-tac.tex b/doc/RefMan-tac.tex
index 9c553473c..b014ded70 100644
--- a/doc/RefMan-tac.tex
+++ b/doc/RefMan-tac.tex
@@ -806,6 +806,10 @@ Applies the conversion tactic {\convtactic} to the
hypotheses \ident$_1$, \ldots, \ident$_n$. The tactic {\convtactic} is
any of the conversion tactics listed in this section.
+If $\ident$_i$ is a local definition, then $\ident$_i$ can be replaced
+by $(Type of \ident$_i)$ to adress not the body but the type of the
+local definition. Example: {\tt Unfold not in (Type of H1) (Type of H3).}
+
\begin{ErrMsgs}
\item \errindex{No such hypothesis} : {\ident}.
\end{ErrMsgs}
@@ -2429,6 +2433,3 @@ user-defined tactics.
%%% TeX-master: "Reference-Manual"
%%% TeX-master: "Reference-Manual"
%%% End:
-
-
-