aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs/pfedit.ml
diff options
context:
space:
mode:
authorGravatar Emilio Jesus Gallego Arias <e+git@x80.org>2018-02-28 21:10:38 +0100
committerGravatar Emilio Jesus Gallego Arias <e+git@x80.org>2018-06-04 18:00:10 +0200
commit31a35fe712a836c90562edebc01bfcf3d1c6646a (patch)
tree754b49914270d0ea219a46dc097c260db95a7d4d /proofs/pfedit.ml
parent9a86eda0766fcc405b57183854c5095cc14cffaa (diff)
[econstr] Remove some Unsafe.to_constr use.
Most of it seems straightforward.
Diffstat (limited to 'proofs/pfedit.ml')
-rw-r--r--proofs/pfedit.ml3
1 files changed, 1 insertions, 2 deletions
diff --git a/proofs/pfedit.ml b/proofs/pfedit.ml
index 03c0969fa..678c3ea3f 100644
--- a/proofs/pfedit.ml
+++ b/proofs/pfedit.ml
@@ -200,8 +200,7 @@ let refine_by_tactic env sigma ty tac =
| [c, _] -> c
| _ -> assert false
in
- let ans = Reductionops.nf_evar sigma ans in
- let ans = EConstr.Unsafe.to_constr ans in
+ let ans = EConstr.to_constr ~abort_on_undefined_evars:false sigma ans in
(** [neff] contains the freshly generated side-effects *)
let neff = Evd.eval_side_effects sigma in
(** Reset the old side-effects *)