aboutsummaryrefslogtreecommitdiff
path: root/doc
diff options
context:
space:
mode:
authormsozeau2009-01-22 14:47:28 +0000
committermsozeau2009-01-22 14:47:28 +0000
commita48e965ab8900eef3d08d6ae814b03bce2df431e (patch)
tree120dd433c22422090a7f645ba797d304a319e2b4 /doc
parent4e13d98beaba323775ab67deb9653504ab4bf91f (diff)
Fixes in the documentation of [dependent induction] and test-suite
scripts. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@11839 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'doc')
-rw-r--r--doc/refman/RefMan-tacex.tex7
1 files changed, 3 insertions, 4 deletions
diff --git a/doc/refman/RefMan-tacex.tex b/doc/refman/RefMan-tacex.tex
index 5da43ec0bb..dbd8634696 100644
--- a/doc/refman/RefMan-tacex.tex
+++ b/doc/refman/RefMan-tacex.tex
@@ -812,8 +812,7 @@ Require Import Coq.Program.Tactics.
Lemma weakening : forall G D tau, term (G ; D) tau ->
forall tau', term (G , tau' ; D) tau.
Proof with simpl in * ; simpl_depind ; auto.
- intros G D tau H.
- dependent induction H generalizing G D.
+ intros G D tau H. dependent induction H generalizing G D ; intros.
\end{coq_example*}
This call to \depind has an additional arguments which is a list of
@@ -845,8 +844,8 @@ Show.
specialize (IHterm G empty).
\end{coq_example}
-Then the automation can find that the needed equality {\tt G = G} to
-narrow the induction hypothesis further. This concludes our example.
+Then the automation can find the needed equality {\tt G = G} to narrow
+the induction hypothesis further. This concludes our example.
\begin{coq_example}
simpl_depind.