aboutsummaryrefslogtreecommitdiff
path: root/proofs
diff options
context:
space:
mode:
Diffstat (limited to 'proofs')
-rw-r--r--proofs/clenv.ml2
-rw-r--r--proofs/tacmach.mli6
2 files changed, 3 insertions, 5 deletions
diff --git a/proofs/clenv.ml b/proofs/clenv.ml
index fd88e3c518..514fc27e89 100644
--- a/proofs/clenv.ml
+++ b/proofs/clenv.ml
@@ -337,7 +337,6 @@ let clenv_pose_metas_as_evars clenv dep_mvs =
let evd = Sigma.Unsafe.of_evar_map clenv.evd in
let Sigma (evar, evd, _) = new_evar (cl_env clenv) evd ~src ty in
let evd = Sigma.to_evar_map evd in
- let evar = EConstr.of_constr evar in
let clenv = clenv_assign mv evar {clenv with evd=evd} in
fold clenv mvs in
fold clenv dep_mvs
@@ -619,7 +618,6 @@ let make_evar_clause env sigma ?len t =
let sigma = Sigma.Unsafe.of_evar_map sigma in
let Sigma (ev, sigma, _) = new_evar ~store env sigma t1 in
let sigma = Sigma.to_evar_map sigma in
- let ev = EConstr.of_constr ev in
let dep = not (noccurn sigma 1 t2) in
let hole = {
hole_evar = ev;
diff --git a/proofs/tacmach.mli b/proofs/tacmach.mli
index 07d02212ca..cfbfe12b17 100644
--- a/proofs/tacmach.mli
+++ b/proofs/tacmach.mli
@@ -67,8 +67,8 @@ val pf_whd_all : goal sigma -> EConstr.constr -> constr
val pf_hnf_constr : goal sigma -> EConstr.constr -> constr
val pf_nf : goal sigma -> EConstr.constr -> constr
val pf_nf_betaiota : goal sigma -> EConstr.constr -> constr
-val pf_reduce_to_quantified_ind : goal sigma -> EConstr.types -> pinductive * types
-val pf_reduce_to_atomic_ind : goal sigma -> EConstr.types -> pinductive * types
+val pf_reduce_to_quantified_ind : goal sigma -> EConstr.types -> pinductive * EConstr.types
+val pf_reduce_to_atomic_ind : goal sigma -> EConstr.types -> pinductive * EConstr.types
val pf_compute : goal sigma -> EConstr.constr -> constr
val pf_unfoldn : (occurrences * evaluable_global_reference) list
-> goal sigma -> EConstr.constr -> constr
@@ -121,7 +121,7 @@ module New : sig
val pf_last_hyp : ([ `NF ], 'r) Proofview.Goal.t -> Context.Named.Declaration.t
val pf_nf_concl : ([ `LZ ], 'r) Proofview.Goal.t -> types
- val pf_reduce_to_quantified_ind : ('a, 'r) Proofview.Goal.t -> EConstr.types -> pinductive * types
+ val pf_reduce_to_quantified_ind : ('a, 'r) Proofview.Goal.t -> EConstr.types -> pinductive * EConstr.types
val pf_hnf_constr : ('a, 'r) Proofview.Goal.t -> EConstr.constr -> types
val pf_hnf_type_of : ('a, 'r) Proofview.Goal.t -> EConstr.constr -> types