aboutsummaryrefslogtreecommitdiff
path: root/vernac/vernacentries.mli
diff options
context:
space:
mode:
authorGaƫtan Gilbert2019-05-21 23:06:40 +0200
committerEnrico Tassi2019-06-04 13:58:43 +0200
commit3b7509b96273f4e412b747e0c55dd193f38fd418 (patch)
treea77d952a62174ded2042cb15ee40abf44c328ca2 /vernac/vernacentries.mli
parent96231a23a9b76b17541572defb6089e23e80c474 (diff)
VernacExtend produces vernac_interp_phase ADT (old name functional_vernac)
+ hide interp_functional_vernac in vernacentries
Diffstat (limited to 'vernac/vernacentries.mli')
-rw-r--r--vernac/vernacentries.mli16
1 files changed, 0 insertions, 16 deletions
diff --git a/vernac/vernacentries.mli b/vernac/vernacentries.mli
index ca3a962319..d94ddc1aaf 100644
--- a/vernac/vernacentries.mli
+++ b/vernac/vernacentries.mli
@@ -51,19 +51,3 @@ val modify_pstate : pstate:Proof_global.stack option -> (pstate:Proof_global.t -
(* Flag set when the test-suite is called. Its only effect to display
verbose information for `Fail` *)
val test_mode : bool ref
-
-(** For mlg *)
-
-type functional_vernac =
- | VtDefault of (unit -> unit)
- | VtCloseProof of (pstate:Proof_global.t -> unit)
- | VtMaybeOpenProof of (unit -> Proof_global.t option)
- | VtOpenProof of (unit -> Proof_global.t)
- | VtModifyProof of (pstate:Proof_global.t -> Proof_global.t)
- | VtReadProofOpt of (pstate:Proof_global.t option -> unit)
- | VtReadProof of (pstate:Proof_global.t -> unit)
-
-val interp_functional_vernac
- : functional_vernac
- -> pstate:Proof_global.stack option
- -> Proof_global.stack option