From 58c70113a815a42593c566f64f2de840fc7e48a1 Mon Sep 17 00:00:00 2001 From: letouzey Date: Tue, 4 Mar 2008 17:33:35 +0000 Subject: migration from Set to Type of FSet/FMap + some dependencies... git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10616 85f007b7-540e-0410-9357-904b9bb8a0f7 --- theories/Sets/Multiset.v | 4 ++-- theories/Sets/Permut.v | 2 +- 2 files changed, 3 insertions(+), 3 deletions(-) (limited to 'theories/Sets') diff --git a/theories/Sets/Multiset.v b/theories/Sets/Multiset.v index 80491c0aa..42130bbb5 100644 --- a/theories/Sets/Multiset.v +++ b/theories/Sets/Multiset.v @@ -16,11 +16,11 @@ Set Implicit Arguments. Section multiset_defs. - Variable A : Set. + Variable A : Type. Variable eqA : A -> A -> Prop. Hypothesis Aeq_dec : forall x y:A, {eqA x y} + {~ eqA x y}. - Inductive multiset : Set := + Inductive multiset : Type := Bag : (A -> nat) -> multiset. Definition EmptyBag := Bag (fun a:A => 0). diff --git a/theories/Sets/Permut.v b/theories/Sets/Permut.v index 7c6b551c6..6c9a064c1 100644 --- a/theories/Sets/Permut.v +++ b/theories/Sets/Permut.v @@ -15,7 +15,7 @@ Section Axiomatisation. - Variable U : Set. + Variable U : Type. Variable op : U -> U -> U. Variable cong : U -> U -> Prop. -- cgit v1.2.3