aboutsummaryrefslogtreecommitdiffhomepage
path: root/vernac/vernacentries.ml
diff options
context:
space:
mode:
authorGravatar Théo Zimmermann <theo.zimmermann@univ-paris-diderot.fr>2017-06-12 11:25:26 +0200
committerGravatar Théo Zimmermann <theo.zimmermann@univ-paris-diderot.fr>2017-06-12 11:25:26 +0200
commit3813ba5229cf42597cd30a08e842e0832e5253cb (patch)
tree0b63fd48d2b021bba3e7518652ac4bc2c5ccc8e4 /vernac/vernacentries.ml
parent6cd14bf253f681d0465f8dce1d84a54a4f104d9c (diff)
Remove Show Thesis command which was never implemented.
Diffstat (limited to 'vernac/vernacentries.ml')
-rw-r--r--vernac/vernacentries.ml4
1 files changed, 0 insertions, 4 deletions
diff --git a/vernac/vernacentries.ml b/vernac/vernacentries.ml
index e0eeaf563..6830a5da1 100644
--- a/vernac/vernacentries.ml
+++ b/vernac/vernacentries.ml
@@ -61,8 +61,6 @@ let show_proof () =
let pprf = Proof.partial_proof p in
Feedback.msg_notice (Pp.prlist_with_sep Pp.fnl Printer.pr_econstr pprf)
-let show_thesis () = CErrors.anomaly (Pp.str "Show Thesis: TODO.")
-
let show_top_evars () =
(* spiwack: new as of Feb. 2010: shows goal evars in addition to non-goal evars. *)
let pfts = get_pftreestate () in
@@ -1843,8 +1841,6 @@ let vernac_show = let open Feedback in function
msg_notice (pr_sequence pr_id (Pfedit.get_all_proof_names()))
| ShowIntros all -> show_intro all
| ShowMatch id -> show_match id
- | ShowThesis -> show_thesis ()
-
let vernac_check_guard () =
let pts = get_pftreestate () in