aboutsummaryrefslogtreecommitdiffhomepage
path: root/doc/refman/CanonicalStructures.tex
diff options
context:
space:
mode:
authorGravatar Guillaume Melquiond <guillaume.melquiond@inria.fr>2015-01-29 15:27:49 +0100
committerGravatar Guillaume Melquiond <guillaume.melquiond@inria.fr>2015-01-29 15:27:49 +0100
commit1dfcae672aa1630bb1fe841bae9321dd9f221fc4 (patch)
tree7346de43dab635ed8d3616b8e7cdf70f9e2ff757 /doc/refman/CanonicalStructures.tex
parentfe038eea4f1c62a209db18fadb69dbab80e16c16 (diff)
Remove spurious "Loading ML file" and "<W> Grammar extension" from the reference manual.
Diffstat (limited to 'doc/refman/CanonicalStructures.tex')
-rw-r--r--doc/refman/CanonicalStructures.tex4
1 files changed, 3 insertions, 1 deletions
diff --git a/doc/refman/CanonicalStructures.tex b/doc/refman/CanonicalStructures.tex
index 7b3bdcf4a..b1c278ced 100644
--- a/doc/refman/CanonicalStructures.tex
+++ b/doc/refman/CanonicalStructures.tex
@@ -305,8 +305,10 @@ canonical structures.
We need some infrastructure for that.
-\begin{coq_example}
+\begin{coq_example*}
Require Import Strings.String.
+\end{coq_example*}
+\begin{coq_example}
Module infrastructure.
Inductive phantom {T : Type} (t : T) : Type := Phantom.
Definition unify {T1 T2} (t1 : T1) (t2 : T2) (s : option string) :=