diff options
Diffstat (limited to 'theories/Sets')
-rw-r--r-- | theories/Sets/Multiset.v | 4 | ||||
-rw-r--r-- | theories/Sets/Permut.v | 2 |
2 files changed, 3 insertions, 3 deletions
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. |