aboutsummaryrefslogtreecommitdiffhomepage
path: root/pretyping
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2016-11-05 18:24:20 +0100
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2017-02-14 17:23:51 +0100
commit214a2ffd2cce3fa24908710af7db528a40345db6 (patch)
tree125f2f5b25e4af803bf95a6edefc51b1555b27a9 /pretyping
parentd528fdaf12b74419c47698cca7c6f1ec762245a3 (diff)
Cbv API using EConstr.
Diffstat (limited to 'pretyping')
-rw-r--r--pretyping/cbv.ml1
-rw-r--r--pretyping/cbv.mli2
-rw-r--r--pretyping/tacred.ml2
3 files changed, 3 insertions, 2 deletions
diff --git a/pretyping/cbv.ml b/pretyping/cbv.ml
index 84bf849e7..a42061f28 100644
--- a/pretyping/cbv.ml
+++ b/pretyping/cbv.ml
@@ -376,6 +376,7 @@ and cbv_norm_value info = function (* reduction under binders *)
(* with profiling *)
let cbv_norm infos constr =
+ let constr = EConstr.Unsafe.to_constr constr in
with_stats (lazy (cbv_norm_term infos (subs_id 0) constr))
type cbv_infos = cbv_value infos
diff --git a/pretyping/cbv.mli b/pretyping/cbv.mli
index 87a03abbd..3d1745767 100644
--- a/pretyping/cbv.mli
+++ b/pretyping/cbv.mli
@@ -19,7 +19,7 @@ open Esubst
type cbv_infos
val create_cbv_infos : RedFlags.reds -> env -> Evd.evar_map -> cbv_infos
-val cbv_norm : cbv_infos -> constr -> constr
+val cbv_norm : cbv_infos -> EConstr.constr -> constr
(***********************************************************************
i This is for cbv debug *)
diff --git a/pretyping/tacred.ml b/pretyping/tacred.ml
index ac2a3bc49..c1e9573d2 100644
--- a/pretyping/tacred.ml
+++ b/pretyping/tacred.ml
@@ -1136,7 +1136,7 @@ let fold_commands cl env sigma c =
(* call by value reduction functions *)
let cbv_norm_flags flags env sigma t =
- cbv_norm (create_cbv_infos flags env sigma) (EConstr.Unsafe.to_constr t)
+ cbv_norm (create_cbv_infos flags env sigma) t
let cbv_beta = cbv_norm_flags beta empty_env
let cbv_betaiota = cbv_norm_flags betaiota empty_env