aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/FSets/FSetFacts.v
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-10-30 15:02:26 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-10-30 15:02:26 +0000
commit5dc1e83de7d933dccd9b8590b77e1c3d4cec593c (patch)
treeadf283c44552ec2d0075bf45be778c24c95e3887 /theories/FSets/FSetFacts.v
parent8787f5b9b1d3191478686c5e01dff6fb9381e508 (diff)
A useless Add Morphism: since Subset is a Setoid Relation, it is also
automatically a Morphism about itself (avoid a warning about redeclared Setoids). git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10277 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/FSets/FSetFacts.v')
-rw-r--r--theories/FSets/FSetFacts.v5
1 files changed, 0 insertions, 5 deletions
diff --git a/theories/FSets/FSetFacts.v b/theories/FSets/FSetFacts.v
index 7eb9b04f6..4de3480d0 100644
--- a/theories/FSets/FSetFacts.v
+++ b/theories/FSets/FSetFacts.v
@@ -469,11 +469,6 @@ unfold Subset; intros s s' H s'' s''' H0 a.
do 2 rewrite diff_iff; intuition.
Qed.
-Add Morphism Subset with signature Subset --> Subset ++> impl as Subset_s_m.
-Proof.
-unfold Subset, impl; auto.
-Qed.
-
(* [fold], [filter], [for_all], [exists_] and [partition] cannot be proved morphism
without additional hypothesis on [f]. For instance: *)