From e4282ea99c664d8d58067bee199cbbcf881b60d5 Mon Sep 17 00:00:00 2001 From: Stephane Glondu Date: Sat, 4 Jul 2009 13:28:35 +0200 Subject: Imported Upstream version 8.2.pl1+dfsg --- theories/FSets/FSetFacts.v | 10 +++++----- 1 file changed, 5 insertions(+), 5 deletions(-) (limited to 'theories/FSets/FSetFacts.v') diff --git a/theories/FSets/FSetFacts.v b/theories/FSets/FSetFacts.v index 1e15d3a1..674caaac 100644 --- a/theories/FSets/FSetFacts.v +++ b/theories/FSets/FSetFacts.v @@ -6,7 +6,7 @@ (* * GNU Lesser General Public License Version 2.1 *) (***********************************************************************) -(* $Id: FSetFacts.v 11720 2008-12-28 07:12:15Z letouzey $ *) +(* $Id: FSetFacts.v 12187 2009-06-13 19:36:59Z msozeau $ *) (** * Finite sets library *) @@ -17,7 +17,7 @@ *) Require Import DecidableTypeEx. -Require Export FSetInterface. +Require Export FSetInterface. Set Implicit Arguments. Unset Strict Implicit. @@ -424,14 +424,14 @@ Add Relation t Subset transitivity proved by Subset_trans as SubsetSetoid. -Instance In_s_m : Morphism (E.eq ==> Subset ++> impl) In | 1. +Instance In_s_m : Morphisms.Morphism (E.eq ==> Subset ++> Basics.impl) In | 1. Proof. simpl_relation. eauto with set. Qed. -Add Morphism Empty with signature Subset --> impl as Empty_s_m. +Add Morphism Empty with signature Subset --> Basics.impl as Empty_s_m. Proof. -unfold Subset, Empty, impl; firstorder. +unfold Subset, Empty, Basics.impl; firstorder. Qed. Add Morphism add with signature E.eq ==> Subset ++> Subset as add_s_m. -- cgit v1.2.3