aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
authorGravatar barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-10-16 16:17:31 +0000
committerGravatar barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-10-16 16:17:31 +0000
commit8fe195799d9bf4eb0c84fad3e9a79b78e6e224ec (patch)
tree647d43ebc553ba697f27d68b658ea26ff44a2492
parent6a66657ecde0b8c16c5ced22ce0f37b86e9c72ee (diff)
typo doc + bug legacy field
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@9243 85f007b7-540e-0410-9357-904b9bb8a0f7
-rw-r--r--contrib/field/field.ml42
-rw-r--r--doc/refman/Polynom.tex8
2 files changed, 5 insertions, 5 deletions
diff --git a/contrib/field/field.ml4 b/contrib/field/field.ml4
index f8f872134..2da5e9fbd 100644
--- a/contrib/field/field.ml4
+++ b/contrib/field/field.ml4
@@ -175,7 +175,7 @@ let guess_theory env evc = function
(* Guesses the type and calls Field_Term with the right theory *)
let field_term l g =
- Coqlib.check_required_library ["Coq";"field";"Field"];
+ Coqlib.check_required_library ["Coq";"field";"LegacyField"];
let env = (pf_env g)
and evc = (project g) in
let th = valueIn (VConstr (guess_theory env evc l))
diff --git a/doc/refman/Polynom.tex b/doc/refman/Polynom.tex
index ee2cf38d3..30dfa93da 100644
--- a/doc/refman/Polynom.tex
+++ b/doc/refman/Polynom.tex
@@ -59,7 +59,7 @@ expression in the \gallina\ language. For example in the ring
\end{verbatim}
\end{quotation}
-\noindent As a ring expression, is has 3 subterms. Give each subterm a
+\noindent As a ring expression, it has 3 subterms. Give each subterm a
number in an arbitrary order:
\begin{tabular}{ccl}
@@ -194,7 +194,7 @@ that can be parameterized. This can be used to improve the handling of
closed expressions when operations are effective. It consists in
introducing a type of \emph{coefficients} and an implementation of the
ring operations, and a morphism from the coefficient type to the ring
-carrier type. The morphism need not be injective, nor surjective. As
+carrier type. The morphism needs not be injective, nor surjective. As
an example, one can consider the real numbers. The set of coefficients
could be the rational numbers, upon which the ring operations can be
implemented. The fact that there exists a morphism is defined by the
@@ -257,7 +257,7 @@ describes their syntax and effects:
setoid. \term$_1$ is a proof that the equality is indeed a setoid
(see {\tt Setoid.Setoid\_Theory}), and \term$_2$ a proof that the
ring operations are morphisms (see {\tt Ring\_theory.ring\_eq\_ext} and
- {\tt Ring\_theory.sring\_eq\_ext}). This modifier need not be used if the
+ {\tt Ring\_theory.sring\_eq\_ext}). This modifier needs not be used if the
setoid and morphisms have been declared.
\item[constants [\ltac]] specifies a tactic expression that, given a term,
returns either an object of the coefficient set that is mapped to
@@ -670,7 +670,7 @@ be significantly less efficient to replace them by tactics using
reflection.
Another idea suggested by Benjamin Werner: reflection could be used to
-couple a external tool (a rewriting program or a model checker) with
+couple an external tool (a rewriting program or a model checker) with
\Coq. We define (in \Coq) a type of terms, a type of \emph{traces},
and prove a correction theorem that states that \emph{replaying
traces} is safe w.r.t some interpretation. Then we let the external