aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs/pfedit.mli
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2015-11-28 19:41:17 +0100
committerGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2015-11-28 19:43:26 +0100
commit90fef3ffd236f2ed5575b0d11a47185185abc75b (patch)
tree2768466af2fc67d61a9e9e94e89fb632d54f3c72 /proofs/pfedit.mli
parent4a11dc25938f3f009e23f1e7c5fe01b2558928c3 (diff)
Univs: correctly register universe binders for lemmas.
Diffstat (limited to 'proofs/pfedit.mli')
-rw-r--r--proofs/pfedit.mli7
1 files changed, 6 insertions, 1 deletions
diff --git a/proofs/pfedit.mli b/proofs/pfedit.mli
index fc521ea43..d0528c9fd 100644
--- a/proofs/pfedit.mli
+++ b/proofs/pfedit.mli
@@ -55,8 +55,10 @@ val delete_all_proofs : unit -> unit
type lemma_possible_guards = Proof_global.lemma_possible_guards
+type universe_binders = Id.t Loc.located list
+
val start_proof :
- Id.t -> goal_kind -> Evd.evar_map -> named_context_val -> constr ->
+ Id.t -> ?pl:universe_binders -> goal_kind -> Evd.evar_map -> named_context_val -> constr ->
?init_tac:unit Proofview.tactic ->
Proof_global.proof_terminator -> unit
@@ -121,6 +123,9 @@ val set_used_variables :
Id.t list -> Context.section_context * (Loc.t * Names.Id.t) list
val get_used_variables : unit -> Context.section_context option
+(** {6 Universe binders } *)
+val get_universe_binders : unit -> universe_binders option
+
(** {6 ... } *)
(** [solve (SelectNth n) tac] applies tactic [tac] to the [n]th
subgoal of the current focused proof or raises a [UserError] if no