aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/dhyp.ml
diff options
context:
space:
mode:
authorGravatar delahaye <delahaye@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-05-03 17:31:07 +0000
committerGravatar delahaye <delahaye@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-05-03 17:31:07 +0000
commitfc38a7d8f3d2a47aa8eee570747568335f3ffa19 (patch)
tree9ddc595a02cf1baaab3e9595d77b0103c80d66bf /tactics/dhyp.ml
parent5b0f516e7e1f6d2ea8ca0485ffe347a613b01a5c (diff)
Ajout du langage de tactiques
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@401 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'tactics/dhyp.ml')
-rw-r--r--tactics/dhyp.ml32
1 files changed, 16 insertions, 16 deletions
diff --git a/tactics/dhyp.ml b/tactics/dhyp.ml
index a21b3e6d7..237af5c06 100644
--- a/tactics/dhyp.ml
+++ b/tactics/dhyp.ml
@@ -111,8 +111,8 @@ open Generic
open Term
open Environ
open Reduction
+open Proof_type
open Rawterm
-open Proof_trees
open Tacmach
open Tactics
open Clenv
@@ -279,17 +279,17 @@ let dHyp id gls = destructHyp false id gls
open Tacinterp
-let _ =
- tacinterp_add
- ("DHyp",(function
- | [Identifier id] -> dHyp id
- | _ -> bad_tactic_args "DHyp"))
+let _=
+ add_tactic "DHyp"
+ (function
+ | [Identifier id] -> dHyp id
+ | _ -> bad_tactic_args "DHyp")
-let _ =
- tacinterp_add
- ("CDHyp",(function
- | [Identifier id] -> cDHyp id
- | _ -> bad_tactic_args "CDHyp"))
+let _=
+ add_tactic "CDHyp"
+ (function
+ | [Identifier id] -> cDHyp id
+ | _ -> bad_tactic_args "CDHyp")
(* [DConcl gls]
@@ -302,11 +302,11 @@ let dConcl gls =
let sorted_ddl = Sort.list (fun dd1 dd2 -> dd1.d_pri > dd2.d_pri) ddl in
tclFIRST (List.map (applyDestructor None false) sorted_ddl) gls
-let _ =
- tacinterp_add
- ("DConcl",(function
- | [] -> dConcl
- | _ -> bad_tactic_args "DConcl"))
+let _=
+ add_tactic "DConcl"
+ (function
+ | [] -> dConcl
+ | _ -> bad_tactic_args "DConcl")
let to2Lists (table : t) = Nbtermdn.to2lists table