aboutsummaryrefslogtreecommitdiffhomepage
path: root/contrib/extraction
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-07-16 15:44:02 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-07-16 15:44:02 +0000
commiteccbf0d1ac7b24cb9e4c1d300f7cb0ccac0f3080 (patch)
tree1d5871343049c1760988f355796a470c8e2e413c /contrib/extraction
parent1d758eca0ab5524a4f24aaa41425716c52618e0c (diff)
Pour ocamlweb
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@2889 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'contrib/extraction')
-rw-r--r--contrib/extraction/extraction.ml6
1 files changed, 3 insertions, 3 deletions
diff --git a/contrib/extraction/extraction.ml b/contrib/extraction/extraction.ml
index 0ac35bda4..ae9034271 100644
--- a/contrib/extraction/extraction.ml
+++ b/contrib/extraction/extraction.ml
@@ -481,7 +481,7 @@ and apply_constant env sp args =
else if la > ls then
let s' = s @ (iterate (fun l -> true :: l) (la-ls) []) in
MLapp (head, extract_real_args env args s')
- else (* la < ls *)
+ else (* [la < ls] *)
let n1 = la
and n2 = ls-la in
let s1,s2 = list_chop n1 s in
@@ -492,7 +492,7 @@ and apply_constant env sp args =
if la >= ls then
let s' = iterate (fun l -> true :: l) (la-ls) [] in
MLapp(head, MLdummy :: (extract_real_args env args s'))
- else (* la < ls *)
+ else (* [la < ls] *)
anonym_lams head (ls-la-1)
(*s Application of an inductive constructor.
@@ -524,7 +524,7 @@ and apply_constructor env cp args =
let mla1 = List.map (ml_lift n2) (extract_real_args env args s1) in
let mla2 = extract_eta_args n2 s2 in
anonym_lams (head (mla1 @ mla2)) n2
- else (* la < params_nb *)
+ else (* [la < params_nb] *)
anonym_lams (head (extract_eta_args ls s)) (ls + params_nb - la)
(*S Extraction of a term. *)