aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
authorGravatar Guillaume Melquiond <guillaume.melquiond@inria.fr>2017-07-28 16:48:25 +0200
committerGravatar Guillaume Melquiond <guillaume.melquiond@inria.fr>2017-07-28 16:48:25 +0200
commiteb483c067985cc9ee7daa160efdc48806eff13e8 (patch)
tree68374614a4fb9f3e8e6172a1fd703ac431150cc8
parent2a7ba998bf7d2c461fdbd8b710b7124395bafaa2 (diff)
Fix some coq-tex errors in the reference manual.
-rw-r--r--doc/refman/Extraction.tex3
-rw-r--r--doc/refman/RefMan-cic.tex3
-rw-r--r--doc/refman/RefMan-sch.tex1
-rw-r--r--doc/refman/RefMan-tacex.tex2
4 files changed, 8 insertions, 1 deletions
diff --git a/doc/refman/Extraction.tex b/doc/refman/Extraction.tex
index fa3d61b1c..a8889be81 100644
--- a/doc/refman/Extraction.tex
+++ b/doc/refman/Extraction.tex
@@ -365,6 +365,9 @@ some specific {\tt Extract Constant} when primitive counterparts exist.
\Example
Typical examples are the following:
+\begin{coq_eval}
+Require Extraction.
+\end{coq_eval}
\begin{coq_example}
Extract Inductive unit => "unit" [ "()" ].
Extract Inductive bool => "bool" [ "true" "false" ].
diff --git a/doc/refman/RefMan-cic.tex b/doc/refman/RefMan-cic.tex
index 96fb1eb75..7a71d6908 100644
--- a/doc/refman/RefMan-cic.tex
+++ b/doc/refman/RefMan-cic.tex
@@ -1425,6 +1425,9 @@ If there is an hypothesis $h:a=b$ in the local context, it can be used for
rewriting not only in logical propositions but also in any type.
% In that case, the term \verb!eq_rec! which was defined as an axiom, is
% now a term of the calculus.
+\begin{coq_eval}
+Require Extraction.
+\end{coq_eval}
\begin{coq_example}
Print eq_rec.
Extraction eq_rec.
diff --git a/doc/refman/RefMan-sch.tex b/doc/refman/RefMan-sch.tex
index d3719bed4..23a1c9b02 100644
--- a/doc/refman/RefMan-sch.tex
+++ b/doc/refman/RefMan-sch.tex
@@ -227,6 +227,7 @@ We define the function \texttt{div2} as follows:
\begin{coq_eval}
Reset Initial.
+Require Import FunInd.
\end{coq_eval}
\begin{coq_example*}
diff --git a/doc/refman/RefMan-tacex.tex b/doc/refman/RefMan-tacex.tex
index 9f4ddc804..cb8f916f1 100644
--- a/doc/refman/RefMan-tacex.tex
+++ b/doc/refman/RefMan-tacex.tex
@@ -849,7 +849,7 @@ Ltac DSimplif trm :=
Ltac Length trm :=
match trm with
| (_ * ?B) => let succ := Length B in constr:(S succ)
- | _ => constr:1
+ | _ => constr:(1)
end.
Ltac assoc := repeat rewrite <- Ass.
\end{coq_example}