aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Setoids
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-12-26 22:26:30 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-12-26 22:26:30 +0000
commit835f581b40183986e76e5e02a26fab05239609c9 (patch)
tree2a42b55f397383aebcb4d6c7950c802c7c51a0eb /theories/Setoids
parentd6615c44439319e99615474cef465d25422a070d (diff)
FMaps: various updates (mostly suggested by P. Casteran)
- New functions: update (a kind of union), restrict (a kind of inter), diff. - New predicat Partition (and Disjoint), many results about Partition. - Equivalence instead of obsolete Setoid_Theory (they are aliases). refl_st, sym_st, trans_st aren't used anymore and marked as obsolete. - Start using Morphism (E.eq==>...) instead of compat_... This change (FMaps only) is incompatible with 8.2betaX, but it's really better now. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@11718 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Setoids')
-rw-r--r--theories/Setoids/Setoid.v37
1 files changed, 23 insertions, 14 deletions
diff --git a/theories/Setoids/Setoid.v b/theories/Setoids/Setoid.v
index 28d8feeae..613cabbd0 100644
--- a/theories/Setoids/Setoid.v
+++ b/theories/Setoids/Setoid.v
@@ -30,20 +30,29 @@ Defined.
(** Some tactics for manipulating Setoid Theory not officially
declared as Setoid. *)
-Ltac trans_st x := match goal with
- | H : Setoid_Theory _ ?eqA |- ?eqA _ _ =>
- apply (Seq_trans _ _ H) with x; auto
- end.
-
-Ltac sym_st := match goal with
- | H : Setoid_Theory _ ?eqA |- ?eqA _ _ =>
- apply (Seq_sym _ _ H); auto
- end.
-
-Ltac refl_st := match goal with
- | H : Setoid_Theory _ ?eqA |- ?eqA _ _ =>
- apply (Seq_refl _ _ H); auto
- end.
+Ltac trans_st x :=
+ idtac "trans_st on Setoid_Theory is OBSOLETE";
+ idtac "use transitivity on Equivalence instead";
+ match goal with
+ | H : Setoid_Theory _ ?eqA |- ?eqA _ _ =>
+ apply (Seq_trans _ _ H) with x; auto
+ end.
+
+Ltac sym_st :=
+ idtac "sym_st on Setoid_Theory is OBSOLETE";
+ idtac "use symmetry on Equivalence instead";
+ match goal with
+ | H : Setoid_Theory _ ?eqA |- ?eqA _ _ =>
+ apply (Seq_sym _ _ H); auto
+ end.
+
+Ltac refl_st :=
+ idtac "refl_st on Setoid_Theory is OBSOLETE";
+ idtac "use reflexivity on Equivalence instead";
+ match goal with
+ | H : Setoid_Theory _ ?eqA |- ?eqA _ _ =>
+ apply (Seq_refl _ _ H); auto
+ end.
Definition gen_st : forall A : Set, Setoid_Theory _ (@eq A).
Proof.