aboutsummaryrefslogtreecommitdiffhomepage
path: root/toplevel/obligations.ml
diff options
context:
space:
mode:
authorGravatar ppedrot <ppedrot@85f007b7-540e-0410-9357-904b9bb8a0f7>2012-06-28 17:52:53 +0000
committerGravatar ppedrot <ppedrot@85f007b7-540e-0410-9357-904b9bb8a0f7>2012-06-28 17:52:53 +0000
commitc62d49b036e48d2753ec4d859e98c4fe027aff66 (patch)
tree54a71005f37fdab2aed118f8a47a67930d8267ce /toplevel/obligations.ml
parent2a167c9a7796939982fa79b4f5adfc7842c97d0e (diff)
Cleaning opening of the standard List module.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@15500 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'toplevel/obligations.ml')
-rw-r--r--toplevel/obligations.ml5
1 files changed, 2 insertions, 3 deletions
diff --git a/toplevel/obligations.ml b/toplevel/obligations.ml
index 0d6bc39f3..4711d9f6d 100644
--- a/toplevel/obligations.ml
+++ b/toplevel/obligations.ml
@@ -25,7 +25,6 @@ open Term
open Sign
open Names
open Evd
-open List
open Pp
open Errors
open Util
@@ -149,7 +148,7 @@ let etype_of_evar evs hyps concl =
| [] ->
let t', s, trans = subst_evar_constr evs n mkVar concl in
subst_vars acc 0 t', s, trans
- in aux [] 0 (rev hyps)
+ in aux [] 0 (List.rev hyps)
open Tacticals
@@ -240,7 +239,7 @@ let eterm_obligations env name evm fs ?status t ty =
in
let evts =
(* Remove existential variables in types and build the corresponding products *)
- fold_right
+ List.fold_right
(fun (id, (n, nstr), ev) l ->
let hyps = Evd.evar_filtered_context ev in
let hyps = trunc_named_context nc_len hyps in