aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-10-13 16:09:17 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-10-13 16:09:17 +0000
commit23c6ebe32a6900d5f70e02279fed48ae74877531 (patch)
tree8e9ecf8b761c620baa81121f75e20d577001018d
parentf7b2d5a90e09242d191a336e13e17cda924a1390 (diff)
Code redondant
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@706 85f007b7-540e-0410-9357-904b9bb8a0f7
-rw-r--r--proofs/refiner.mli6
-rw-r--r--proofs/tacmach.ml4
2 files changed, 4 insertions, 6 deletions
diff --git a/proofs/refiner.mli b/proofs/refiner.mli
index 8546b0c73..be59f5685 100644
--- a/proofs/refiner.mli
+++ b/proofs/refiner.mli
@@ -26,12 +26,6 @@ val add_tactic : string -> (tactic_arg list -> tactic) -> unit
val overwriting_add_tactic : string -> (tactic_arg list -> tactic) -> unit
val lookup_tactic : string -> (tactic_arg list) -> tactic
-val hide_tactic :
- string -> (tactic_arg list -> tactic) -> (tactic_arg list -> tactic)
-
-val overwrite_hidden_tactic :
- string -> (tactic_arg list -> tactic) -> (tactic_arg list -> tactic)
-
val refiner : rule -> tactic
val context : ctxtty -> tactic
val vernac_tactic : tactic_expression -> tactic
diff --git a/proofs/tacmach.ml b/proofs/tacmach.ml
index 0d4d279d5..88ca18f1c 100644
--- a/proofs/tacmach.ml
+++ b/proofs/tacmach.ml
@@ -328,10 +328,14 @@ let tactic_com_bind_list_list tac args gl =
(* Functions for hiding the implementation of a tactic. *)
(********************************************************)
+(* hide_tactic s tac pr registers a tactic s under the name s *)
+
let hide_tactic s tac =
add_tactic s tac;
(fun args -> vernac_tactic(s,args))
+(* overwriting_register_tactic s tac pr registers a tactic s under the
+ name s even if a tactic of the same name is already registered *)
let overwrite_hidden_tactic s tac =
overwriting_add_tactic s tac;