aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs/goal.mli
diff options
context:
space:
mode:
authorGravatar ppedrot <ppedrot@85f007b7-540e-0410-9357-904b9bb8a0f7>2013-03-12 20:59:33 +0000
committerGravatar ppedrot <ppedrot@85f007b7-540e-0410-9357-904b9bb8a0f7>2013-03-12 20:59:33 +0000
commit198586739090e63ad65051449f1a80f751c4c08b (patch)
tree9247931c1505bcf8549d5daa4547b227ebe7ae47 /proofs/goal.mli
parent7c281301637f783beaec858a5fee665e99a6813b (diff)
Allowing different types of, not to be mixed, generic Stores through
functor application. Rewritten the interface btw. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@16267 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'proofs/goal.mli')
-rw-r--r--proofs/goal.mli5
1 files changed, 2 insertions, 3 deletions
diff --git a/proofs/goal.mli b/proofs/goal.mli
index 49667879b..6b587959a 100644
--- a/proofs/goal.mli
+++ b/proofs/goal.mli
@@ -28,7 +28,6 @@ val pr_goal : goal -> Pp.std_ppcmds
(* [advance sigma g] returns [Some g'] if [g'] is undefined and
is the current avatar of [g] (for instance [g] was changed by [clear]
into [g']). It returns [None] if [g] has been (partially) solved. *)
-open Store.Field
val advance : Evd.evar_map -> goal -> goal option
@@ -189,7 +188,7 @@ module V82 : sig
val concl : Evd.evar_map -> goal -> Term.constr
(* Access to ".evar_extra" *)
- val extra : Evd.evar_map -> goal -> Store.t
+ val extra : Evd.evar_map -> goal -> Evd.Store.t
(* Old style filtered_context primitive *)
val filtered_context : Evd.evar_map -> goal -> Sign.named_context
@@ -200,7 +199,7 @@ module V82 : sig
val mk_goal : Evd.evar_map ->
Environ.named_context_val ->
Term.constr ->
- Store.t ->
+ Evd.Store.t ->
goal * Term.constr * Evd.evar_map
(* Equality function on goals *)