aboutsummaryrefslogtreecommitdiffhomepage
path: root/kernel/nativeconv.ml
diff options
context:
space:
mode:
authorGravatar Maxime Dénès <mail@maximedenes.fr>2015-01-16 22:17:03 +0100
committerGravatar Maxime Dénès <mail@maximedenes.fr>2015-01-17 08:02:45 +0100
commit9f5586d88880cbb98c92edfe9c33c76564f1a19c (patch)
tree6de2a171eff5706b0e4ce9268554b84a922f12b3 /kernel/nativeconv.ml
parent4985f0ff99278beb3b934f86edf1398659c611a8 (diff)
Make native compiler handle universe polymorphic definitions.
One remaining issue: aliased constants raise an anomaly when some unsubstituted universe variables remain. VM may suffer from the same problem.
Diffstat (limited to 'kernel/nativeconv.ml')
-rw-r--r--kernel/nativeconv.ml81
1 files changed, 39 insertions, 42 deletions
diff --git a/kernel/nativeconv.ml b/kernel/nativeconv.ml
index 8930250fc..75a3fc458 100644
--- a/kernel/nativeconv.ml
+++ b/kernel/nativeconv.ml
@@ -16,17 +16,17 @@ open Nativecode
(** This module implements the conversion test by compiling to OCaml code *)
-let rec conv_val env pb lvl v1 v2 cu =
- if v1 == v2 then cu
+let rec conv_val env pb lvl cu v1 v2 =
+ if v1 == v2 then ()
else
match kind_of_value v1, kind_of_value v2 with
| Vaccu k1, Vaccu k2 ->
- conv_accu env pb lvl k1 k2 cu
+ conv_accu env pb lvl cu k1 k2
| Vfun f1, Vfun f2 ->
let v = mk_rel_accu lvl in
- conv_val env CONV (lvl+1) (f1 v) (f2 v) cu
+ conv_val env CONV (lvl+1) cu (f1 v) (f2 v)
| Vconst i1, Vconst i2 ->
- if Int.equal i1 i2 then cu else raise NotConvertible
+ if not (Int.equal i1 i2) then raise NotConvertible
| Vblock b1, Vblock b2 ->
let n1 = block_size b1 in
let n2 = block_size b2 in
@@ -34,79 +34,76 @@ let rec conv_val env pb lvl v1 v2 cu =
raise NotConvertible;
let rec aux lvl max b1 b2 i cu =
if Int.equal i max then
- conv_val env CONV lvl (block_field b1 i) (block_field b2 i) cu
+ conv_val env CONV lvl cu (block_field b1 i) (block_field b2 i)
else
- let cu =
- conv_val env CONV lvl (block_field b1 i) (block_field b2 i) cu in
- aux lvl max b1 b2 (i+1) cu in
+ (conv_val env CONV lvl cu (block_field b1 i) (block_field b2 i);
+ aux lvl max b1 b2 (i+1) cu)
+ in
aux lvl (n1-1) b1 b2 0 cu
| Vfun f1, _ ->
- conv_val env CONV lvl v1 (fun x -> v2 x) cu
+ conv_val env CONV lvl cu v1 (fun x -> v2 x)
| _, Vfun f2 ->
- conv_val env CONV lvl (fun x -> v1 x) v2 cu
+ conv_val env CONV lvl cu (fun x -> v1 x) v2
| _, _ -> raise NotConvertible
-and conv_accu env pb lvl k1 k2 cu =
+and conv_accu env pb lvl cu k1 k2 =
let n1 = accu_nargs k1 in
let n2 = accu_nargs k2 in
if not (Int.equal n1 n2) then raise NotConvertible;
if Int.equal n1 0 then
conv_atom env pb lvl (atom_of_accu k1) (atom_of_accu k2) cu
else
- let cu = conv_atom env pb lvl (atom_of_accu k1) (atom_of_accu k2) cu in
- List.fold_right2 (conv_val env CONV lvl) (args_of_accu k1) (args_of_accu k2) cu
+ (conv_atom env pb lvl (atom_of_accu k1) (atom_of_accu k2) cu;
+ List.iter2 (conv_val env CONV lvl cu) (args_of_accu k1) (args_of_accu k2))
and conv_atom env pb lvl a1 a2 cu =
- if a1 == a2 then cu
+ if a1 == a2 then ()
else
match a1, a2 with
| Arel i1, Arel i2 ->
- if not (Int.equal i1 i2) then raise NotConvertible;
- cu
+ if not (Int.equal i1 i2) then raise NotConvertible
| Aind ind1, Aind ind2 ->
- if not (eq_ind ind1 ind2) then raise NotConvertible;
- cu
+ if not (eq_puniverses eq_ind ind1 ind2) then raise NotConvertible
| Aconstant c1, Aconstant c2 ->
- if not (eq_constant c1 c2) then raise NotConvertible;
- cu
+ if not (eq_puniverses eq_constant c1 c2) then raise NotConvertible
| Asort s1, Asort s2 ->
- check_sort_cmp_universes env pb s1 s2 cu; cu
+ check_sort_cmp_universes env pb s1 s2 cu
| Avar id1, Avar id2 ->
- if not (Id.equal id1 id2) then raise NotConvertible;
- cu
+ if not (Id.equal id1 id2) then raise NotConvertible
| Acase(a1,ac1,p1,bs1), Acase(a2,ac2,p2,bs2) ->
if not (eq_ind a1.asw_ind a2.asw_ind) then raise NotConvertible;
- let cu = conv_accu env CONV lvl ac1 ac2 cu in
+ conv_accu env CONV lvl cu ac1 ac2;
let tbl = a1.asw_reloc in
let len = Array.length tbl in
- if Int.equal len 0 then conv_val env CONV lvl p1 p2 cu
- else
- let cu = conv_val env CONV lvl p1 p2 cu in
+ if Int.equal len 0 then conv_val env CONV lvl cu p1 p2
+ else begin
+ conv_val env CONV lvl cu p1 p2;
let max = len - 1 in
- let rec aux i cu =
+ let rec aux i =
let tag,arity = tbl.(i) in
let ci =
if Int.equal arity 0 then mk_const tag
else mk_block tag (mk_rels_accu lvl arity) in
let bi1 = bs1 ci and bi2 = bs2 ci in
- if Int.equal i max then conv_val env CONV (lvl + arity) bi1 bi2 cu
- else aux (i+1) (conv_val env CONV (lvl + arity) bi1 bi2 cu) in
- aux 0 cu
+ if Int.equal i max then conv_val env CONV (lvl + arity) cu bi1 bi2
+ else (conv_val env CONV (lvl + arity) cu bi1 bi2; aux (i+1)) in
+ aux 0
+ end
| Afix(t1,f1,rp1,s1), Afix(t2,f2,rp2,s2) ->
if not (Int.equal s1 s2) || not (Array.equal Int.equal rp1 rp2) then raise NotConvertible;
- if f1 == f2 then cu
+ if f1 == f2 then ()
else conv_fix env lvl t1 f1 t2 f2 cu
| (Acofix(t1,f1,s1,_) | Acofixe(t1,f1,s1,_)),
(Acofix(t2,f2,s2,_) | Acofixe(t2,f2,s2,_)) ->
if not (Int.equal s1 s2) then raise NotConvertible;
- if f1 == f2 then cu
+ if f1 == f2 then ()
else
if not (Int.equal (Array.length f1) (Array.length f2)) then raise NotConvertible
else conv_fix env lvl t1 f1 t2 f2 cu
| Aprod(_,d1,c1), Aprod(_,d2,c2) ->
- let cu = conv_val env CONV lvl d1 d2 cu in
+ conv_val env CONV lvl cu d1 d2;
let v = mk_rel_accu lvl in
- conv_val env pb (lvl + 1) (d1 v) (d2 v) cu
+ conv_val env pb (lvl + 1) cu (d1 v) (d2 v)
| _, _ -> raise NotConvertible
(* Precondition length t1 = length f1 = length f2 = length t2 *)
@@ -115,13 +112,13 @@ and conv_fix env lvl t1 f1 t2 f2 cu =
let max = len - 1 in
let fargs = mk_rels_accu lvl len in
let flvl = lvl + len in
- let rec aux i cu =
- let cu = conv_val env CONV lvl t1.(i) t2.(i) cu in
+ let rec aux i =
+ conv_val env CONV lvl cu t1.(i) t2.(i);
let fi1 = napply f1.(i) fargs in
let fi2 = napply f2.(i) fargs in
- if Int.equal i max then conv_val env CONV flvl fi1 fi2 cu
- else aux (i+1) (conv_val env CONV flvl fi1 fi2 cu) in
- aux 0 cu
+ if Int.equal i max then conv_val env CONV flvl cu fi1 fi2
+ else (conv_val env CONV flvl cu fi1 fi2; aux (i+1)) in
+ aux 0
let native_conv pb sigma env t1 t2 =
if !Flags.no_native_compiler then begin
@@ -144,7 +141,7 @@ let native_conv pb sigma env t1 t2 =
let time_info = Format.sprintf "Evaluation done in %.5f@." (t1 -. t0) in
if !Flags.debug then Pp.msg_debug (Pp.str time_info);
(* TODO change 0 when we can have deBruijn *)
- ignore(conv_val env pb 0 !rt1 !rt2 (Environ.universes env))
+ conv_val env pb 0 (Environ.universes env) !rt1 !rt2
end
| _ -> anomaly (Pp.str "Compilation failure")