aboutsummaryrefslogtreecommitdiffhomepage
path: root/doc/RefMan-tacex.tex
diff options
context:
space:
mode:
authorGravatar filliatr <filliatr@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-04-06 16:08:55 +0000
committerGravatar filliatr <filliatr@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-04-06 16:08:55 +0000
commitc411b544498a1114c21deb2186f29ddc37b9611e (patch)
tree4b9bc201ec3c643e33fdd8d2b6f36c448c686fc1 /doc/RefMan-tacex.tex
parent7d4466949d2ae0d65ebe22b96dccc51d7aea2b01 (diff)
mise a jour V7
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@8171 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'doc/RefMan-tacex.tex')
-rw-r--r--doc/RefMan-tacex.tex7
1 files changed, 3 insertions, 4 deletions
diff --git a/doc/RefMan-tacex.tex b/doc/RefMan-tacex.tex
index 274802056..8e30077fb 100644
--- a/doc/RefMan-tacex.tex
+++ b/doc/RefMan-tacex.tex
@@ -518,7 +518,7 @@ Inductive Type formula :=
| f_or : formula -> formula -> formula
| f_not : formula -> formula (* unary constructor *)
| f_true : formula (* 0-ary constructor *)
-| f_const : Prop -> formula. (* contructor for constants *)
+| f_const : Prop -> formula (* contructor for constants *).
Fixpoint interp_f [f:formula] : Prop :=
Cases f of
@@ -528,7 +528,6 @@ Fixpoint interp_f [f:formula] : Prop :=
| f_true => True
| (f_const c) => c
end.
-
Goal A/\(A\/True)/\~B/\(A <-> A).
Quote interp_f.
\end{coq_example}
@@ -541,7 +540,7 @@ return the corresponding constructor (here \texttt{f\_const}) applied
to the term.
\begin{ErrMsgs}
-\item \errindex{Quote: not a simple fixpoint}
+\item \errindex{Quote: not a simple fixpoint} \\
Happens when \texttt{Quote} is not able to perform inversion properly.
\end{ErrMsgs}
@@ -576,7 +575,7 @@ Inductive Set formula :=
| f_or : formula -> formula -> formula
| f_not : formula -> formula
| f_true : formula
-| f_atom : index -> formula. (* contructor for variables *)
+| f_atom : index -> formula.
\end{coq_example*}
\texttt{index} is defined in module \texttt{Quote}. Equality on that