aboutsummaryrefslogtreecommitdiffhomepage
path: root/doc
diff options
context:
space:
mode:
authorGravatar barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-10-20 10:08:51 +0000
committerGravatar barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-10-20 10:08:51 +0000
commitbba1bdbe36d454ffb387e182998ccf174d177628 (patch)
tree789acbd737b0cd21080de1d60b0f73b2a3df12ef /doc
parent7c58006651a73c74bbb5564ee79d9ff8d59eb3d8 (diff)
*** empty log message ***
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4675 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'doc')
-rw-r--r--doc/memo-v8.tex2
-rw-r--r--doc/syntax-v8.tex89
2 files changed, 54 insertions, 37 deletions
diff --git a/doc/memo-v8.tex b/doc/memo-v8.tex
index 23e5b6708..8d116de26 100644
--- a/doc/memo-v8.tex
+++ b/doc/memo-v8.tex
@@ -257,7 +257,7 @@ occurence numbers of this term, the occurence numbers are put after
the term itself. This applies to tactic \TERM{pattern} and also
\TERM{unfold}
\begin{transbox}
-\TRANS{Pattern 1 2 (f x) 3 4 d}{pattern (f x) 1 2, d 3 4}
+\TRANS{Pattern 1 2 (f x) 3 4 d y z}{pattern (f x at 1 2) (d at 3 4) y z}
\end{transbox}
\section{Main changes in vernacular commands w.r.t. V7}
diff --git a/doc/syntax-v8.tex b/doc/syntax-v8.tex
index 41e5eb62a..e06fa48a3 100644
--- a/doc/syntax-v8.tex
+++ b/doc/syntax-v8.tex
@@ -682,47 +682,50 @@ has the keyword to be associated to \KWD{let} or to tactic \TERM{simpl} ?
\subsection{Other tactics}
-TODO
-
\begin{rules}
\EXTNT{simple-tactic}
- \TERM{rewrite}
-\nlsep \TERM{replace}
-\nlsep \TERM{symplify_eq}
-\nlsep \TERM{discriminate}
-\nlsep \TERM{injection}
-\nlsep \TERM{conditional rewrite}
-\nlsep \TERM{dependent rewrite}
-\nlsep \TERM{absurd}
+ \TERM{rewrite} ~\NT{orient} ~\NT{constr-with-bindings}
+ ~\OPTGR{\KWD{in}~\NT{ident}}
+\nlsep \TERM{replace} ~\tacconstr ~\KWD{with} ~\tacconstr
+ ~\OPTGR{\KWD{in}~\NT{ident}}
+\nlsep \TERM{replace} ~\OPT{\NT{orient}} ~\tacconstr
+ ~\OPTGR{\KWD{in}~\NT{ident}}
+\nlsep \TERM{symplify_eq} ~\OPT{\NT{quantified-hyp}}
+\nlsep \TERM{discriminate} ~\OPT{\NT{quantified-hyp}}
+\nlsep \TERM{injection} ~\OPT{\NT{quantified-hyp}}
+\nlsep \TERM{conditional}~\NT{tactic}~\TERM{rewrite}~NT{orient}
+ ~\NT{constr-with-bindings}~\OPTGR{\KWD{in}~\NT{ident}
+\nlsep \TERM{dependent}~\TERM{rewrite}~\NT{orient}~\NT{ident}
+\nlsep \TERM{cutrewrite}~\NT{orient}~\tacconstr}
+ ~\OPTGR{\KWD{in}~\NT{ident}}
+\nlsep \TERM{absurd} ~\tacconstr
\nlsep \TERM{contradiction}
-\nlsep \TERM{autorewrite}
-\nlsep \TERM{hint rewrite}
-\nlsep \TERM{refine}
-\nlsep \TERM{setoid_replace}
-\nlsep \TERM{setoid_rewrite}
-\nlsep \TERM{add setoid}
-\nlsep \TERM{add morphism}
-\nlsep \TERM{inversion}
-\nlsep \TERM{simple}~\TERM{inversion}
-\nlsep \TERM{derive}~\TERM{inversion_clear}
-\nlsep \TERM{derive}~\TERM{inversion}
-\nlsep \TERM{derive}~\TERM{dependent}~\TERM{inversion}
-\nlsep \TERM{derive}~\TERM{dependent}~\TERM{inversion_clear}
-\nlsep \TERM{subst}
+\nlsep \TERM{autorewrite}~\TERM{[}~\PLUS{\NT{ident}}~\TERM{]}
+ ~\OPTGR{\KWD{using}~\NT{tactic}}
+\nlsep \TERM{refine}~\tacconstr
+\nlsep \TERM{setoid_replace} ~\tacconstr ~\KWD{with} ~\tacconstr
+\nlsep \TERM{setoid_rewrite} ~\NT{orient} ~\tacconstr
+\nlsep \TERM{subst} ~\STAR{\NT{ident}}
%% eqdecide.ml4
-\nlsep \TERM{decide}~\TERM{equality}
-\nlsep \TERM{compare}
+\nlsep \TERM{decide}~\TERM{equality} ~\OPTGR{\tacconstr~\tacconstr}
+\nlsep \TERM{compare}~\tacconstr~\tacconstr
%% eauto
-\nlsep \TERM{eexact}
-\nlsep \TERM{eapply}
-\nlsep \TERM{prolog}
-\nlsep \TERM{eauto}
-\nlsep \TERM{eautod}
+\nlsep \TERM{eexact}~\tacconstr
+\nlsep \TERM{eapply}~\NT{constr-with-bindings}
+\nlsep \TERM{prolog}~\TERM{[}~\STAR{\tacconstr}~\TERM{]}
+ ~\NT{quantified-hyp}
+\nlsep \TERM{eauto}~\OPT{\NT{quantified-hyp}}~\OPT{\NT{quantified-hyp}}
+ ~\NT{hintbases}
+\nlsep \TERM{eautod}~\OPT{\NT{quantified-hyp}}~\OPT{\NT{quantified-hyp}}
+ ~\NT{hintbases}
%% tauto
\nlsep \TERM{tauto}
\nlsep \TERM{simplif}
-\nlsep \TERM{intuition}
-\nlsep \TERM{linearintuition}
+\nlsep \TERM{intuition}~\OPT{\NTL{tactic}{0}}
+\nlsep \TERM{linearintuition}~\OPT{\NT{int}}
+\SEPDEF
+\DEFNT{orient}
+ \KWD{$\rightarrow$}~\mid~\KWD{$\leftarrow$}
\end{rules}
\section{Grammar of commands}
@@ -1021,6 +1024,21 @@ $$
\TERM{Ltac}~\NT{ident}~\STAR{\NT{name}}~\KWD{:=}~\NT{tactic}
\nlsep \TERM{Debug}~\TERM{On}
\nlsep \TERM{Debug}~\TERM{Off}
+%% TODO: vernac
+\nlsep \TERM{add}~\TERM{setoid}~\tacconstr~\tacconstr~\tacconstr
+\nlsep \TERM{add}~\TERM{morphism}~\tacconstr~\KWD{:}~\NT{ident}
+\nlsep \TERM{derive}~\TERM{inversion_clear}
+ ~\OPT{\NT{int}}~\NT{ident}~\NT{ident}
+\nlsep \TERM{derive}~\TERM{inversion_clear}
+ ~\NT{ident}~\KWD{with}~\tacconstr~\OPTGR{\TERM{Sort}~\NT{sort}}
+\nlsep \TERM{derive}~\TERM{inversion}
+ ~\OPT{\NT{int}}~\NT{ident}~\NT{ident}
+\nlsep \TERM{derive}~\TERM{inversion}
+ ~\NT{ident}~\KWD{with}~\tacconstr~\OPTGR{\TERM{Sort}~\NT{sort}}
+\nlsep \TERM{derive}~\TERM{dependent}~\TERM{inversion_clear}
+ ~\NT{ident}~\KWD{with}~\tacconstr~\OPTGR{\TERM{Sort}~\NT{sort}}
+\nlsep \TERM{derive}~\TERM{dependent}~\TERM{inversion}
+ ~\NT{ident}~\KWD{with}~\tacconstr~\OPTGR{\TERM{Sort}~\NT{sort}}
\end{rules}
@@ -1069,6 +1087,8 @@ $$
\nlsep \TERM{Hint}~\TERM{Destruct}~\NT{destruct-loc}~\NT{int}
~\NT{ident}~\NT{constr}~\KWD{$\Rightarrow$}~\NT{tactic}
\nlsep \TERM{Hint}~\NT{hint}~\OPT{\NT{hintbases}}
+%% TODO
+\nlsep \TERM{Hint}~\TERM{rewrite} ...
%% PrintConstr not documented
\end{rules}
@@ -1089,9 +1109,6 @@ $$
\DEFNT{hintbases}
\KWD{:}~\PLUS{\NT{ident}}
\SEPDEF
-\DEFNT{orient}
- \KWD{$\rightarrow$}~\mid~\KWD{$\leftarrow$}
-\SEPDEF
\DEFNT{destruct-loc}
\TERM{Conclusion}
\nlsep \OPT{\TERM{Discardable}}~\TERM{Hypothesis}