aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/setoid_replace.mli
diff options
context:
space:
mode:
Diffstat (limited to 'tactics/setoid_replace.mli')
-rw-r--r--tactics/setoid_replace.mli8
1 files changed, 5 insertions, 3 deletions
diff --git a/tactics/setoid_replace.mli b/tactics/setoid_replace.mli
index 1eb0141c6..244e02dd4 100644
--- a/tactics/setoid_replace.mli
+++ b/tactics/setoid_replace.mli
@@ -12,6 +12,7 @@ open Term
open Proof_type
open Topconstr
open Names
+open Termops
type relation =
{ rel_a: constr ;
@@ -40,7 +41,7 @@ type morphism_signature = (bool option * constr_expr) list * constr_expr
val pr_morphism_signature : morphism_signature -> Pp.std_ppcmds
val register_replace : (tactic option -> constr -> constr -> tactic) -> unit
-val register_general_rewrite : (bool -> int list -> constr -> tactic) -> unit
+val register_general_rewrite : (bool -> occurrences -> constr -> tactic) -> unit
val print_setoids : unit -> unit
@@ -58,9 +59,10 @@ val setoid_replace_in :
identifier -> constr option -> constr -> constr -> new_goals:constr list ->
tactic
-val general_s_rewrite : bool -> int list -> constr -> new_goals:constr list -> tactic
+val general_s_rewrite :
+ bool -> occurrences -> constr -> new_goals:constr list -> tactic
val general_s_rewrite_in :
- identifier -> bool -> int list -> constr -> new_goals:constr list -> tactic
+ identifier -> bool -> occurrences -> constr -> new_goals:constr list -> tactic
val setoid_reflexivity : tactic
val setoid_symmetry : tactic