aboutsummaryrefslogtreecommitdiffhomepage
path: root/contrib/first-order/rules.mli
diff options
context:
space:
mode:
authorGravatar corbinea <corbinea@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-04-26 15:14:15 +0000
committerGravatar corbinea <corbinea@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-04-26 15:14:15 +0000
commitb1901a4f1278465179718d614b3d26b19eefcd75 (patch)
tree4ab7f21b4754dfacb9a6ed69a518c8e1a12b8093 /contrib/first-order/rules.mli
parent0cf3324183974110b5fd0b0317b014b1e4629fe3 (diff)
bugfix in Ground tactic
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@3957 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'contrib/first-order/rules.mli')
-rw-r--r--contrib/first-order/rules.mli7
1 files changed, 5 insertions, 2 deletions
diff --git a/contrib/first-order/rules.mli b/contrib/first-order/rules.mli
index 98dc01bbe..ee224bc54 100644
--- a/contrib/first-order/rules.mli
+++ b/contrib/first-order/rules.mli
@@ -11,13 +11,16 @@
open Term
open Tacmach
open Names
+open Libnames
type hptac= Sequent.t -> (Sequent.t -> tactic) -> Formula.counter -> tactic
-type lhptac= identifier -> hptac
+type lhptac= global_reference -> hptac
val wrap : int -> bool -> hptac
+val clear_global: global_reference -> tactic
+
val axiom_tac : constr -> Sequent.t -> tactic
val and_tac : hptac
@@ -44,7 +47,7 @@ val ll_atom_tac : constr -> lhptac
val ll_false_tac : lhptac
-val left_false_tac : identifier -> tactic
+val left_false_tac : global_reference -> tactic
val ll_ind_tac : inductive -> constr list -> lhptac