aboutsummaryrefslogtreecommitdiffhomepage
path: root/doc/refman
diff options
context:
space:
mode:
authorGravatar fbesson <fbesson@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-07-02 13:24:47 +0000
committerGravatar fbesson <fbesson@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-07-02 13:24:47 +0000
commit3bf96f48739699da368bb872663945ebdb2d78a4 (patch)
tree7d29f2a7a70a3b345bdc3587fe2563d6a586576d /doc/refman
parent7f110df7d7ff6a4d43f3c8d19305b20e24f4800e (diff)
Improved robustness of micromega parser. Proof search of Micromega test-suites is now bounded -- ensure termination
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@11200 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'doc/refman')
-rw-r--r--doc/refman/Micromega.tex4
1 files changed, 2 insertions, 2 deletions
diff --git a/doc/refman/Micromega.tex b/doc/refman/Micromega.tex
index 11e3e8cce..234d51134 100644
--- a/doc/refman/Micromega.tex
+++ b/doc/refman/Micromega.tex
@@ -17,11 +17,11 @@ Load the {\tt Psatz} module ({\tt Require Psatz}.). This module defines the tac
\begin{itemize}
\item The {\tt psatzl} tactic solves linear goals using an embedded (naive) linear programming prover \emph{i.e.},
fourier elimination.
- \item The {\tt psatz} tactic solves polynomial goals using an external prover {\tt cspd}\footnote{Source and binaries can be found at \url{https://projects.coin-or.org/Csdp}}. Note that the {\tt csdp} driver is generating
+ \item The {\tt psatz} tactic solves polynomial goals using John Harrison's Hol light driver to the external prover {\tt cspd}\footnote{Source and binaries can be found at \url{https://projects.coin-or.org/Csdp}}. Note that the {\tt csdp} driver is generating
a \emph{proof cache} thus allowing to rerun scripts even without {\tt csdp}.
\item The {\tt lia} (linear integer arithmetic) tactic is specialised to solve linear goals over $\mathbb{Z}$.
It extends {\tt psatzl Z} and exploits the discreetness of $\mathbb{Z}$.
- \item The {\tt sos} tactic is another driver to the {\tt csdp} prover. In theory, it is less general than
+ \item The {\tt sos} tactic is another Hol light driver to the {\tt csdp} prover. In theory, it is less general than
{\tt psatz}. In practice, even when {\tt psatz} fails, it can be worth a try -- see
Section~\ref{sec:psatz-back} for details.
\end{itemize}