aboutsummaryrefslogtreecommitdiff
path: root/API
diff options
context:
space:
mode:
authorMaxime Dénès2017-07-19 16:22:48 +0200
committerMaxime Dénès2017-07-19 16:22:48 +0200
commit4d4ec6a095d01b6117ac3682d8a7882b1a2520e7 (patch)
treed9ad4f412a3d3889ce869a4c0aecbc9dc098271a /API
parente273ff57ef82e81ab6b6309584a7d496ae4659c1 (diff)
parentab53757a3bf57ced503023f3cf9dea5b5503dfea (diff)
Merge PR #770: [proof] Move bullets to their own module.
Diffstat (limited to 'API')
-rw-r--r--API/API.ml1
-rw-r--r--API/API.mli6
2 files changed, 6 insertions, 1 deletions
diff --git a/API/API.ml b/API/API.ml
index 093ca97f80..32c664d7b1 100644
--- a/API/API.ml
+++ b/API/API.ml
@@ -79,6 +79,7 @@ module Nametab = Nametab
module Vernacentries = Vernacentries
module Mltop = Mltop
module Goal = Goal
+module Proof_bullet = Proof_bullet
module Proof_global = Proof_global
module Proof = Proof
module Smartlocate = Smartlocate
diff --git a/API/API.mli b/API/API.mli
index e8418552c4..b1a746e028 100644
--- a/API/API.mli
+++ b/API/API.mli
@@ -3449,6 +3449,11 @@ sig
end
end
+module Proof_bullet :
+sig
+ val get_default_goal_selector : unit -> Vernacexpr.goal_selector
+end
+
module Proof_global :
sig
type proof_mode = Proof_global.proof_mode = {
@@ -3483,7 +3488,6 @@ sig
(unit Proofview.tactic -> Proof.proof -> Proof.proof) -> unit
val compact_the_proof : unit -> unit
val register_proof_mode : proof_mode -> unit
- val get_default_goal_selector : unit -> Vernacexpr.goal_selector
exception NoCurrentProof
val give_me_the_proof : unit -> Proof.proof