aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
authorGravatar Maxime Dénès <mail@maximedenes.fr>2017-11-06 11:22:39 +0100
committerGravatar Maxime Dénès <mail@maximedenes.fr>2017-11-06 11:22:39 +0100
commitdc6f4b07c38b416b1771bf7436af9303f25f0c1e (patch)
treec02a44b299fbf5f534477229d9db7feaebfe754a
parentc757ec96e2f281e618c297ffc6098aacf1e3f399 (diff)
parent3e5ba8bb1188e9c0f59c04bd0e8fa7c9ff5bc52b (diff)
Merge PR #6063: Finish removing Show Goal uid
-rw-r--r--intf/vernacexpr.ml1
-rw-r--r--printing/ppvernac.ml2
-rw-r--r--printing/printer.ml11
-rw-r--r--printing/printer.mli1
-rw-r--r--proofs/goal.ml1
-rw-r--r--proofs/goal.mli3
-rw-r--r--vernac/vernacentries.ml1
7 files changed, 1 insertions, 19 deletions
diff --git a/intf/vernacexpr.ml b/intf/vernacexpr.ml
index ea412a7d6..9aef4b131 100644
--- a/intf/vernacexpr.ml
+++ b/intf/vernacexpr.ml
@@ -39,7 +39,6 @@ type goal_reference =
| OpenSubgoals
| NthGoal of int
| GoalId of Id.t
- | GoalUid of goal_identifier
type printable =
| PrintTables
diff --git a/printing/ppvernac.ml b/printing/ppvernac.ml
index d1158b3d6..143f9ddcc 100644
--- a/printing/ppvernac.ml
+++ b/printing/ppvernac.ml
@@ -574,7 +574,7 @@ open Decl_kinds
| OpenSubgoals -> mt ()
| NthGoal n -> spc () ++ int n
| GoalId id -> spc () ++ pr_id id
- | GoalUid n -> spc () ++ str n in
+ in
let pr_showable = function
| ShowGoal n -> keyword "Show" ++ pr_goal_reference n
| ShowProof -> keyword "Show Proof"
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
diff --git a/printing/printer.mli b/printing/printer.mli
index 658ea6060..f55206f0d 100644
--- a/printing/printer.mli
+++ b/printing/printer.mli
@@ -201,7 +201,6 @@ val pr_assumptionset :
env -> Term.types ContextObjectMap.t -> Pp.t
val pr_goal_by_id : Id.t -> Pp.t
-val pr_goal_by_uid : string -> Pp.t
type printer_pr = {
pr_subgoals : ?pr_first:bool -> Pp.t option -> evar_map -> evar list -> Goal.goal list -> int list -> goal list -> goal list -> Pp.t;
diff --git a/proofs/goal.ml b/proofs/goal.ml
index 7d830146f..61f3e4a02 100644
--- a/proofs/goal.ml
+++ b/proofs/goal.ml
@@ -21,7 +21,6 @@ type goal = Evd.evar
let pr_goal e = str "GOAL:" ++ Pp.int (Evar.repr e)
let uid e = string_of_int (Evar.repr e)
-let get_by_uid u = Evar.unsafe_of_int (int_of_string u)
(* Layer to implement v8.2 tactic engine ontop of the new architecture.
Types are different from what they used to be due to a change of the
diff --git a/proofs/goal.mli b/proofs/goal.mli
index 6d3ec8bd4..ad968cdfb 100644
--- a/proofs/goal.mli
+++ b/proofs/goal.mli
@@ -15,9 +15,6 @@ type goal = Evar.t
(* Gives a unique identifier to each goal. The identifier is
guaranteed to contain no space. *)
val uid : goal -> string
-(* Returns the goal (even if it has been partially solved)
- corresponding to a unique identifier obtained by {!uid}. *)
-val get_by_uid : string -> goal
(* Debugging help *)
val pr_goal : goal -> Pp.t
diff --git a/vernac/vernacentries.ml b/vernac/vernacentries.ml
index f83546ea6..41f63644d 100644
--- a/vernac/vernacentries.ml
+++ b/vernac/vernacentries.ml
@@ -1853,7 +1853,6 @@ let vernac_show = let open Feedback in function
| OpenSubgoals -> pr_open_subgoals ()
| NthGoal n -> pr_nth_open_subgoal n
| GoalId id -> pr_goal_by_id id
- | GoalUid id -> pr_goal_by_uid id
in
msg_notice info
| ShowProof -> show_proof ()