aboutsummaryrefslogtreecommitdiff
path: root/doc/tutorial
diff options
context:
space:
mode:
authorEmilio Jesus Gallego Arias2017-05-17 20:55:32 +0200
committerEmilio Jesus Gallego Arias2017-05-23 01:37:24 +0200
commit3c0d8d08bda81b9fbd7210e4e352a08bbe8219e8 (patch)
tree22c4573182302aa493a18f275833e2fdf78306c9 /doc/tutorial
parent11851daee3a14f784cc2a30536a8f69be62c4f62 (diff)
[vernac] Remove `Save.` command.
It has been deprecated for a while in favor of `Qed`.
Diffstat (limited to 'doc/tutorial')
-rw-r--r--doc/tutorial/Tutorial.tex8
1 files changed, 3 insertions, 5 deletions
diff --git a/doc/tutorial/Tutorial.tex b/doc/tutorial/Tutorial.tex
index 0d537256bb..30b6304c16 100644
--- a/doc/tutorial/Tutorial.tex
+++ b/doc/tutorial/Tutorial.tex
@@ -385,13 +385,11 @@ apply H; [ assumption | apply H0; assumption ].
Let us now save lemma \verb:distr_impl::
\begin{coq_example}
-Save.
+Qed.
\end{coq_example}
-Here \verb:Save: needs no argument, since we gave the name \verb:distr_impl:
-in advance;
-it is however possible to override the given name by giving a different
-argument to command \verb:Save:.
+Here \verb:Qed: needs no argument, since we gave the name \verb:distr_impl:
+in advance.
Actually, such an easy combination of tactics \verb:intro:, \verb:apply:
and \verb:assumption: may be found completely automatically by an automatic