aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs/goal.ml
diff options
context:
space:
mode:
authorGravatar ppedrot <ppedrot@85f007b7-540e-0410-9357-904b9bb8a0f7>2013-10-05 19:53:10 +0000
committerGravatar ppedrot <ppedrot@85f007b7-540e-0410-9357-904b9bb8a0f7>2013-10-05 19:53:10 +0000
commit49d4bfb1f40cbcb06902094d5f6b7a6340eae1dd (patch)
tree848dd45c82a65547dd025d67d866c3d39e819ab1 /proofs/goal.ml
parent65eec025bc0b581fae1af78f18d1a8666b76e69b (diff)
Removing dubious use of evarmap manipulating functions in printing
related code. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@16851 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'proofs/goal.ml')
-rw-r--r--proofs/goal.ml9
1 files changed, 3 insertions, 6 deletions
diff --git a/proofs/goal.ml b/proofs/goal.ml
index 0eacde878..48cce3fa7 100644
--- a/proofs/goal.ml
+++ b/proofs/goal.ml
@@ -171,10 +171,7 @@ module Refinable = struct
(* a pessimistic (i.e : there won't be many positive answers) filter
over evar_maps, acting only on undefined evars *)
let evar_map_filter_undefined f evm =
- Evd.fold_undefined
- (fun ev evi r -> if f ev evi then Evd.add r ev evi else r)
- evm
- Evd.empty
+ Evar.Map.filter f (Evd.undefined_map evm)
(* Union, sorted in decreasing order, of two lists of evars in decreasing order. *)
let rec fusion l1 l2 = match l1 , l2 with
@@ -193,7 +190,7 @@ module Refinable = struct
post_defs
in
(* [delta_evars] in the shape of a list of [evar]-s*)
- let delta_list = List.map fst (Evd.to_list delta_evars) in
+ let delta_list = List.map fst (Evar.Map.bindings delta_evars) in
(* The variables in [myevars] are supposed to be stored
in decreasing order. Breaking this invariant might cause
many things to go wrong. *)
@@ -229,7 +226,7 @@ module Refinable = struct
let constr_of_open_constr handle check_type (evars, c) env rdefs gl info =
let delta = update_handle handle !rdefs evars in
- rdefs := Evd.fold (fun ev evi evd -> Evd.add evd ev evi) delta !rdefs;
+ rdefs := Evar.Map.fold (fun ev evi evd -> Evd.add evd ev evi) delta !rdefs;
if check_type then with_type c (Evd.evar_concl (content !rdefs gl)) env rdefs gl info
else c