aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/setoid_replace.mli
diff options
context:
space:
mode:
authorGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-04-12 16:01:36 +0000
committerGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-04-12 16:01:36 +0000
commit1ea4a8d26516af14670cc677a5a0fce04b90caf7 (patch)
treef97ad5097f4a5ef3eb3c71e2affb646f22d3ec51 /tactics/setoid_replace.mli
parentdf77da121b86c64a91ea729f39afc92f10676893 (diff)
Adding 'at' to rewrite, as it is already implemented in setoid_rewrite.
Uses setoid_rewrite even if rewriting with leibniz if there are specified occurences, maybe a combination of pattern and rewrite could be done instead. Correct spelling of occurrences. Coq does not compile with this patch, the next one will make it compile again. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10781 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'tactics/setoid_replace.mli')
-rw-r--r--tactics/setoid_replace.mli6
1 files changed, 3 insertions, 3 deletions
diff --git a/tactics/setoid_replace.mli b/tactics/setoid_replace.mli
index 2dd153b3f..1eb0141c6 100644
--- a/tactics/setoid_replace.mli
+++ b/tactics/setoid_replace.mli
@@ -40,7 +40,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 -> constr -> tactic) -> unit
+val register_general_rewrite : (bool -> int list -> constr -> tactic) -> unit
val print_setoids : unit -> unit
@@ -58,9 +58,9 @@ val setoid_replace_in :
identifier -> constr option -> constr -> constr -> new_goals:constr list ->
tactic
-val general_s_rewrite : bool -> constr -> new_goals:constr list -> tactic
+val general_s_rewrite : bool -> int list -> constr -> new_goals:constr list -> tactic
val general_s_rewrite_in :
- identifier -> bool -> constr -> new_goals:constr list -> tactic
+ identifier -> bool -> int list -> constr -> new_goals:constr list -> tactic
val setoid_reflexivity : tactic
val setoid_symmetry : tactic