aboutsummaryrefslogtreecommitdiffhomepage
path: root/printing/printer.ml
diff options
context:
space:
mode:
authorGravatar Gaëtan Gilbert <gaetan.gilbert@skyskimmer.net>2017-11-04 15:59:31 +0100
committerGravatar Gaëtan Gilbert <gaetan.gilbert@skyskimmer.net>2017-11-04 15:59:31 +0100
commit3e5ba8bb1188e9c0f59c04bd0e8fa7c9ff5bc52b (patch)
tree105c101301a9628159896c636395b66f17220cda /printing/printer.ml
parentf281a8a88e8fc7c41cc5680db2443d9da33b47b7 (diff)
Finish removing Show Goal uid
Diffstat (limited to 'printing/printer.ml')
-rw-r--r--printing/printer.ml11
1 files changed, 0 insertions, 11 deletions
diff --git a/printing/printer.ml b/printing/printer.ml
index c6650ea3b..70e96722d 100644
--- a/printing/printer.ml
+++ b/printing/printer.ml
@@ -838,17 +838,6 @@ let pr_goal_by_id id =
pr_selected_subgoal (pr_id id) sigma g)
with Not_found -> user_err Pp.(str "No such goal.")
-let pr_goal_by_uid uid =
- let p = Proof_global.give_me_the_proof () in
- let g = Goal.get_by_uid uid in
- let pr gs =
- v 0 (str "goal / evar " ++ str uid ++ str " is:" ++ cut ()
- ++ pr_goal gs)
- in
- try
- Proof.in_proof p (fun sigma -> pr {it=g;sigma=sigma;})
- with Not_found -> user_err Pp.(str "Invalid goal identifier.")
-
(* Elementary tactics *)
let pr_prim_rule = function