aboutsummaryrefslogtreecommitdiffhomepage
path: root/doc
diff options
context:
space:
mode:
authorGravatar pboutill <pboutill@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-09-28 16:27:28 +0000
committerGravatar pboutill <pboutill@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-09-28 16:27:28 +0000
commit56a2994e2ecc931836fb4ef8b2bdb027a705cfcd (patch)
tree14d0bb8cebf6e81059baf64b01ee0d03f8f6521a /doc
parente09064ff153ee9f909e8c2c1ee2aaa249b324a78 (diff)
Minor fixes of 'make doc'
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@13472 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'doc')
-rw-r--r--doc/faq/FAQ.tex4
-rwxr-xr-xdoc/stdlib/Library.tex1
2 files changed, 3 insertions, 2 deletions
diff --git a/doc/faq/FAQ.tex b/doc/faq/FAQ.tex
index baf3d4991..0e5b00d37 100644
--- a/doc/faq/FAQ.tex
+++ b/doc/faq/FAQ.tex
@@ -1688,7 +1688,7 @@ Lemma Rwf : well_founded R.
\item Define the step function (which needs proofs that recursive
calls are on smaller arguments).
-\begin{coq_example*}
+\begin{verbatim}
Definition split (l : list nat)
: {l1: list nat | R l1 l} * {l2 : list nat | R l2 l}
:= (* ... *) .
@@ -1698,7 +1698,7 @@ Definition merge_step (l : list nat) (f: forall l':list nat, R l' l -> list nat)
let (l1,H1) := lH1 in
let (l2,H2) := lH2 in
concat (f l1 H1) (f l2 H2).
-\end{coq_example*}
+\end{verbatim}
\item Define the recursive function by fixpoint on the step function.
diff --git a/doc/stdlib/Library.tex b/doc/stdlib/Library.tex
index 02dc61bfe..cb32adfcf 100755
--- a/doc/stdlib/Library.tex
+++ b/doc/stdlib/Library.tex
@@ -3,6 +3,7 @@
\usepackage[utf8x]{inputenc}
\usepackage[T1]{fontenc}
\usepackage{fullpage}
+\usepackage{amsfonts}
\usepackage[color]{../../coqdoc}
\input{../common/version}