aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs/proofview.mli
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <mattam@mattam.org>2014-06-18 17:16:59 +0200
committerGravatar Matthieu Sozeau <mattam@mattam.org>2014-06-18 17:21:21 +0200
commit23f4804b50307766219392229757e75da9aa41d9 (patch)
tree4df833759b600b1a3d638bdbc65cf5060eb3e24f /proofs/proofview.mli
parent77839ae306380e99a8ceac0bf26ff86ec9159346 (diff)
Proofs now take and return an evar_universe_context, simplifying interfaces
and avoiding explicit substitutions and merging of contexts, e.g. in obligations.ml. The context produced by typechecking a statement is passed in the proof, allowing the universe name context to be correctly folded as well. Mainly an API cleanup.
Diffstat (limited to 'proofs/proofview.mli')
-rw-r--r--proofs/proofview.mli6
1 files changed, 3 insertions, 3 deletions
diff --git a/proofs/proofview.mli b/proofs/proofview.mli
index c27e4ba1a..f959513d4 100644
--- a/proofs/proofview.mli
+++ b/proofs/proofview.mli
@@ -37,11 +37,11 @@ type entry
(* Initialises a proofview, the argument is a list of environement,
conclusion types, creating that many initial goals. *)
-val init : Evd.evar_map -> (Environ.env * Term.types Univ.in_universe_context_set) list -> entry * proofview
+val init : Evd.evar_map -> (Environ.env * Term.types) list -> entry * proofview
type telescope =
| TNil
- | TCons of Environ.env * Term.types Univ.in_universe_context_set * (Term.constr -> telescope)
+ | TCons of Environ.env * Term.types * (Term.constr -> telescope)
(* Like [init], but goals are allowed to be depedenent on one
another. Dependencies between goals is represented with the type
@@ -57,7 +57,7 @@ val finished : proofview -> bool
val return : proofview -> Evd.evar_map
val partial_proof : entry -> proofview -> constr list
-val initial_goals : entry -> (constr * types Univ.in_universe_context_set) list
+val initial_goals : entry -> (constr * types) list
val emit_side_effects : Declareops.side_effects -> proofview -> proofview
(*** Focusing operations ***)