aboutsummaryrefslogtreecommitdiffhomepage
path: root/doc/refman/RefMan-tac.tex
diff options
context:
space:
mode:
authorGravatar gareuselesinge <gareuselesinge@85f007b7-540e-0410-9357-904b9bb8a0f7>2013-08-08 18:52:02 +0000
committerGravatar gareuselesinge <gareuselesinge@85f007b7-540e-0410-9357-904b9bb8a0f7>2013-08-08 18:52:02 +0000
commit0a329ae992825e98314ba4c6c4c6152d60b2bbeb (patch)
tree68d3810338a72046f259e2ae0a44a3f316b9c0cd /doc/refman/RefMan-tac.tex
parentb2f2727670853183bfbcbafb9dc19f0f71494a7b (diff)
Manual fixed w.r.t. STM
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@16675 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'doc/refman/RefMan-tac.tex')
-rw-r--r--doc/refman/RefMan-tac.tex2
1 files changed, 1 insertions, 1 deletions
diff --git a/doc/refman/RefMan-tac.tex b/doc/refman/RefMan-tac.tex
index a091da2df..805b2cee0 100644
--- a/doc/refman/RefMan-tac.tex
+++ b/doc/refman/RefMan-tac.tex
@@ -882,7 +882,7 @@ Qed.
Goal forall n:nat, n = 0 -> n = 0.
intros [ | ] H.
Show 2.
-Undo.
+Undo 2.
intros [ | ]; intros H.
Show 2.
\end{coq_example}