aboutsummaryrefslogtreecommitdiff
path: root/kernel
diff options
context:
space:
mode:
authorMaxime Dénès2019-04-14 14:02:16 +0200
committerMaxime Dénès2019-04-15 15:28:09 +0200
commit7205996bf25a542224c815b38f92da0ffef76b5d (patch)
tree4853a361c9a1efe4f3d4163f47c0fa4cc514ce05 /kernel
parent137e8b1636fa0b25c232ed42944ecaed058732ee (diff)
[native compiler] Remove unused universe argument in Lmakeblock
Diffstat (limited to 'kernel')
-rw-r--r--kernel/nativecode.ml2
-rw-r--r--kernel/nativelambda.ml14
-rw-r--r--kernel/nativelambda.mli2
3 files changed, 9 insertions, 9 deletions
diff --git a/kernel/nativecode.ml b/kernel/nativecode.ml
index c879cab9df..375f3184de 100644
--- a/kernel/nativecode.ml
+++ b/kernel/nativecode.ml
@@ -1274,7 +1274,7 @@ let ml_of_instance instance u =
| Lint tag -> MLapp(MLprimitive Mk_int, [|MLint tag|])
- | Lmakeblock (prefix,(cn,_u),_,args) ->
+ | Lmakeblock (prefix,cn,_,args) ->
let args = Array.map (ml_of_lam env l) args in
MLconstruct(prefix,cn,args)
| Luint i -> MLapp(MLprimitive Mk_uint, [|MLuint i|])
diff --git a/kernel/nativelambda.ml b/kernel/nativelambda.ml
index 02b5043135..40948244fb 100644
--- a/kernel/nativelambda.ml
+++ b/kernel/nativelambda.ml
@@ -40,7 +40,7 @@ type lambda =
| Lfix of (int array * (string * inductive) array * int) * fix_decl
| Lcofix of int * fix_decl
| Lint of int (* a constant constructor *)
- | Lmakeblock of prefix * pconstructor * int * lambda array
+ | Lmakeblock of prefix * constructor * int * lambda array
(* prefix, constructor Name.t, constructor tag, arguments *)
(* A fully applied non-constant constructor *)
| Luint of Uint63.t
@@ -342,11 +342,11 @@ let expand_constructor prefix cstr tag nparams arity =
Llam(ids, Lmakeblock (prefix, cstr, tag, args))
(* [nparams] is the number of parameters still expected *)
-let makeblock env cn u tag nparams arity args =
+let makeblock env cn tag nparams arity args =
let nargs = Array.length args in
if nparams > 0 || nargs < arity then
let prefix = get_mind_prefix env (fst (fst cn)) in
- mkLapp (expand_constructor prefix (cn,u) tag nparams arity) args
+ mkLapp (expand_constructor prefix cn tag nparams arity) args
else
(* The constructor is fully applied *)
if Int.equal arity 0 then Lint tag
@@ -356,7 +356,7 @@ let makeblock env cn u tag nparams arity args =
Lval (Nativevalues.mk_block tag args)
else
let prefix = get_mind_prefix env (fst (fst cn)) in
- Lmakeblock(prefix, (cn,u), tag, args)
+ Lmakeblock(prefix, cn, tag, args)
(* Translation of constants *)
@@ -584,13 +584,13 @@ and lambda_of_app cache env sigma f args =
let prefix = get_const_prefix env kn in
mkLapp (Lconst (prefix, (kn,u))) (lambda_of_args cache env sigma 0 args)
end
- | Construct (c,u) ->
+ | Construct (c,_) ->
let tag, nparams, arity = Cache.get_construct_info cache env c in
let nargs = Array.length args in
if nparams < nargs then (* got all parameters *)
let args = lambda_of_args cache env sigma nparams args in
- makeblock env c u tag 0 arity args
- else makeblock env c u tag (nparams - nargs) arity empty_args
+ makeblock env c tag 0 arity args
+ else makeblock env c tag (nparams - nargs) arity empty_args
| _ ->
let f = lambda_of_constr cache env sigma f in
let args = lambda_of_args cache env sigma 0 args in
diff --git a/kernel/nativelambda.mli b/kernel/nativelambda.mli
index c357819da5..093665df9b 100644
--- a/kernel/nativelambda.mli
+++ b/kernel/nativelambda.mli
@@ -34,7 +34,7 @@ type lambda =
| Lfix of (int array * (string * inductive) array * int) * fix_decl
| Lcofix of int * fix_decl
| Lint of int (* a constant constructor *)
- | Lmakeblock of prefix * pconstructor * int * lambda array
+ | Lmakeblock of prefix * constructor * int * lambda array
(* prefix, constructor Name.t, constructor tag, arguments *)
(* A fully applied non-constant constructor *)
| Luint of Uint63.t