aboutsummaryrefslogtreecommitdiffhomepage
path: root/doc/refman/RefMan-pro.tex
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-07-07 15:37:23 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-07-07 15:37:23 +0000
commitb00500d44818b6d182bd4e8b233bc963bfbf5505 (patch)
tree9302596762b3aa1a89e9498f8542cfffc3da9e33 /doc/refman/RefMan-pro.tex
parent165d5c2e7c8bd4402f33987ad3fe91d92fe0b808 (diff)
Documentation Declare Implicit Tactic, Print Canonical Projections, ... + légère restructuration autour de Proof with et Hint Rewrite + maj crédits
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@9030 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'doc/refman/RefMan-pro.tex')
-rw-r--r--doc/refman/RefMan-pro.tex17
1 files changed, 5 insertions, 12 deletions
diff --git a/doc/refman/RefMan-pro.tex b/doc/refman/RefMan-pro.tex
index 7565612d1..ddfce775d 100644
--- a/doc/refman/RefMan-pro.tex
+++ b/doc/refman/RefMan-pro.tex
@@ -163,28 +163,21 @@ as a {\tt Theorem}, the name {\ident} is known at all section levels:
current section.
\end{Variants}
-\subsection{\tt Proof {\term}.}\comindex{Proof}
+\subsection{\tt Proof {\term}.}
+\comindex{Proof}
+\label{BeginProof}
This command applies in proof editing mode. It is equivalent to {\tt
exact {\term}; Save.} That is, you have to give the full proof in
one gulp, as a proof term (see section \ref{exact}).
-\begin{Variants}
-
-\item{\tt Proof.}
+\variant {\tt Proof.}
Is a noop which is useful to delimit the sequence of tactic commands
which start a proof, after a {\tt Theorem} command. It is a good
practice to use {\tt Proof.} as an opening parenthesis, closed in
the script with a closing {\tt Qed.}
-\item{\tt Proof with {\tac}.}
-
- This command may be used to start a proof. It defines a default
- tactic to be used each time a tactic command is ended by
- ``\verb#...#''. In this case the tactic command typed by the user is
- equivalent to \emph{command};{\tac}.
-
-\end{Variants}
+\SeeAlso {\tt Proof with {\tac}.} in section~\ref{ProofWith}.
\subsection{\tt Abort.}
\comindex{Abort}