aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2015-02-16 11:30:24 +0100
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2015-02-16 12:22:53 +0100
commit100d50d7cde05334940378a1e6483cae975b93a5 (patch)
tree8d1bd6ff514d724ed9d117bb7dad71f254d7dd91
parent4e6c9891140932f452bb5ac8960d597b0b5fde1d (diff)
Documenting "induction t in ctx" when ctx contains an hyp not mentioning t.
-rw-r--r--doc/refman/RefMan-tac.tex16
1 files changed, 13 insertions, 3 deletions
diff --git a/doc/refman/RefMan-tac.tex b/doc/refman/RefMan-tac.tex
index ee40a0d51..c2407dce2 100644
--- a/doc/refman/RefMan-tac.tex
+++ b/doc/refman/RefMan-tac.tex
@@ -1789,9 +1789,19 @@ induction n.
\item \texttt{induction {\term} in {\occgoalset}}
This syntax is used for selecting which occurrences of {\term} the
- induction has to be carried on. The {\tt in \occgoalset} clause is an
- occurrence clause whose syntax and behavior is described in
- Section~\ref{Occurrences_clauses}.
+ induction has to be carried on. The {\tt in \occgoalset} clause is
+ an occurrence clause whose syntax and behavior is described in
+ Section~\ref{Occurrences_clauses}. If variables or hypotheses not
+ mentioning {\term} in their type are listed in {\occgoalset}, those
+ are generalized as well in the statement to prove.
+
+\Example
+
+\begin{coq_example}
+Lemma comm x y : x + y = y + x.
+induction y in x |- *.
+Show 2.
+\end{coq_example}
\item {\tt induction {\term$_1$} with {\bindinglist$_1$}
as {\disjconjintropattern} %% eqn:{\namingintropattern}