aboutsummaryrefslogtreecommitdiffhomepage
path: root/doc/RefMan-tac.tex
diff options
context:
space:
mode:
authorGravatar barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7>2004-01-14 16:52:06 +0000
committerGravatar barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7>2004-01-14 16:52:06 +0000
commite92027584f4134f4fa89a77a752bf28aedd9c44a (patch)
tree0eefd0cf15a2f05fed2f49bf8b1ff26796fdf834 /doc/RefMan-tac.tex
parent4ba765fe88d88e5765d6058b7d366e03318b789a (diff)
ajout d'une passe de latex our avoir un index correct
+ quelques petites retouches sur la doc git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@8476 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'doc/RefMan-tac.tex')
-rw-r--r--doc/RefMan-tac.tex13
1 files changed, 7 insertions, 6 deletions
diff --git a/doc/RefMan-tac.tex b/doc/RefMan-tac.tex
index 0b9f7b7b5..43c6f965b 100644
--- a/doc/RefMan-tac.tex
+++ b/doc/RefMan-tac.tex
@@ -1281,7 +1281,7 @@ Proof c.
This tactic applies to any goal. If the variables {\ident$_1$} and
{\ident$_2$} of the goal have an inductive type, then this tactic
performs double induction on these variables. For instance, if the
-current goal is \verb+(n,m:nat)(P n m)+ then, {\tt double induction n
+current goal is \verb+forall n m:nat, P n m+ then, {\tt double induction n
m} yields the four cases with their respective inductive hypotheses.
In particular the case for \verb+(P (S n) (S m))+ with the induction
hypotheses \verb+(P (S n) m)+ and \verb+(m:nat)(P n m)+ (hence
@@ -1653,10 +1653,10 @@ introduced hypothesis.
\item{\tt injection}\tacindex{injection}
- If the current goal is of the form {\tt
- \verb=~={\term$_1$}={\term$_2$}}, the tactic computes the head
- normal form of the goal and then behaves as the sequence: {\tt
- unfold not; intro {\ident}; injection {\ident}}.
+ If the current goal is of the form {\term$_1$} {\tt <>} {\term$_2$},
+ the tactic computes the head normal form of the goal and then
+ behaves as the sequence: {\tt unfold not; intro {\ident}; injection
+ {\ident}}.
\ErrMsg \errindex{goal does not satisfy the expected preconditions}
\end{Variants}
@@ -1678,7 +1678,8 @@ latter is first introduced in the local context using
\texttt{intros until \ident}.
\begin{Variants}
-\item \texttt{simplify\_eq} \num\\
+\item \texttt{simplify\_eq} \num
+
This does the same thing as \texttt{intros until \num} then
\texttt{simplify\_eq \ident} where {\ident} is the identifier for the last
introduced hypothesis.