aboutsummaryrefslogtreecommitdiff
path: root/kernel
diff options
context:
space:
mode:
authorregisgia2010-08-27 09:32:10 +0000
committerregisgia2010-08-27 09:32:10 +0000
commitd12a7327183054ee5c45f5327105738dcd31c548 (patch)
treee80757e364007666f1c4205c0599db41143dda2e /kernel
parent129a58c5dd2403263b8285f345b3a5e41d480b78 (diff)
* checker/SafeTyping kernel/SafeTyping:
Fix typos. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@13380 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'kernel')
-rw-r--r--kernel/safe_typing.ml4
1 files changed, 2 insertions, 2 deletions
diff --git a/kernel/safe_typing.ml b/kernel/safe_typing.ml
index e384e510ba..504bfab04b 100644
--- a/kernel/safe_typing.ml
+++ b/kernel/safe_typing.ml
@@ -906,7 +906,7 @@ end = struct
(get_table : unit -> table)) =
(* We use an integer as a key inside the table. *)
let counter = ref 0 in
- (* ... but it is wrap inside a [constr_substituted]. *)
+ (* ... but it is wrapped inside a [constr_substituted]. *)
let key_as_constr key = Declarations.from_val (Term.mkRel key) in
(* During the traversal, the table is implemented by a list
@@ -929,7 +929,7 @@ end = struct
let lightened_library = traverse_library encode_const_body library in
(lightened_library, get_table ())
- (* Loading is also a traversing that decode the embedded keys that
+ (* Loading is also a traversing that decodes the embedded keys that
are inside the [lightened_library]. If the [load_proof] flag is
set, we lookup inside the table to graft the
[constr_substituted]. Otherwise, we set the [const_body] field