diff options
author | letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2010-06-18 16:19:43 +0000 |
---|---|---|
committer | letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2010-06-18 16:19:43 +0000 |
commit | 7dac84295d86c425c301641c55683894f5c22c55 (patch) | |
tree | 3c51b40f7a02569fc678b19eb5a8295e232f20b9 /theories/FSets | |
parent | 405885980b4a7a7eeb8d26cd5a7ad0f132ac6388 (diff) |
fsetdec: a forgotten Set instead of Type was breaking discard_nonFset (fix #2281)
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@13163 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/FSets')
-rw-r--r-- | theories/FSets/FSetDecide.v | 2 |
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/FSets/FSetDecide.v b/theories/FSets/FSetDecide.v index 2769c7611..cc78fdb4d 100644 --- a/theories/FSets/FSetDecide.v +++ b/theories/FSets/FSetDecide.v @@ -416,7 +416,7 @@ the above form: propositions of interest. *) Inductive FSet_elt_Prop : Prop -> Prop := - | eq_Prop : forall (S : Set) (x y : S), + | eq_Prop : forall (S : Type) (x y : S), FSet_elt_Prop (x = y) | eq_elt_prop : forall x y, FSet_elt_Prop (E.eq x y) |