diff options
| author | Enrico Tassi | 2019-05-22 18:30:31 +0200 |
|---|---|---|
| committer | Enrico Tassi | 2019-06-04 13:58:43 +0200 |
| commit | d77604cb06fcc8e8f38ef979627aa7a7138ef0f2 (patch) | |
| tree | f1b96b0faf85806d7e926e0216f94515d5cddf3a | |
| parent | 2ebd73901edb94030aa804572cbe86d486ca6732 (diff) | |
[vernac] remove VtMaybeOpenProof
| -rw-r--r-- | coqpp/coqpp_main.ml | 1 | ||||
| -rw-r--r-- | vernac/vernacentries.ml | 4 | ||||
| -rw-r--r-- | vernac/vernacextend.ml | 1 | ||||
| -rw-r--r-- | vernac/vernacextend.mli | 1 |
4 files changed, 0 insertions, 7 deletions
diff --git a/coqpp/coqpp_main.ml b/coqpp/coqpp_main.ml index d6ae0a7d6f..d5aedfcbb1 100644 --- a/coqpp/coqpp_main.ml +++ b/coqpp/coqpp_main.ml @@ -359,7 +359,6 @@ let print_atts_right fmt = function let understand_state = function | "close_proof" -> "VtCloseProof", false - | "maybe_open_proof" -> "VtMaybeOpenProof", true | "open_proof" -> "VtOpenProof", true | "proof" -> "VtModifyProof", false | "proof_opt_query" -> "VtReadProofOpt", false diff --git a/vernac/vernacentries.ml b/vernac/vernacentries.ml index 949ddfc3ee..da9fa35202 100644 --- a/vernac/vernacentries.ml +++ b/vernac/vernacentries.ml @@ -2304,10 +2304,6 @@ let vernac_interp_phase c ~pstate = vernac_require_open_proof ~pstate (fun ~pstate -> f ~pstate:(Proof_global.get_current_pstate pstate); Proof_global.discard_current pstate) - | VtMaybeOpenProof f -> - let proof = f () in - let pstate = maybe_push ~ontop:pstate proof in - pstate | VtOpenProof f -> Some (push ~ontop:pstate (f ())) | VtModifyProof f -> diff --git a/vernac/vernacextend.ml b/vernac/vernacextend.ml index cf704206af..2d3443d30a 100644 --- a/vernac/vernacextend.ml +++ b/vernac/vernacextend.ml @@ -56,7 +56,6 @@ type vernac_classification = vernac_type * vernac_when type vernac_interp_phase = | 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) diff --git a/vernac/vernacextend.mli b/vernac/vernacextend.mli index 4d885a3afc..f06f31d45b 100644 --- a/vernac/vernacextend.mli +++ b/vernac/vernacextend.mli @@ -74,7 +74,6 @@ type vernac_classification = vernac_type * vernac_when type vernac_interp_phase = | 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) |
