aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/MSets/MSetList.v
diff options
context:
space:
mode:
authorGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-11-15 00:15:42 +0000
committerGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-11-15 00:15:42 +0000
commit77ba6079eef1099a34bfcff01fe36298392e3fdf (patch)
tree466868e3c5c3ffb57d32083ca2a51067e4926d09 /theories/MSets/MSetList.v
parent600e73d2522599fd600ab717410254565d57236b (diff)
Fix [Instance: forall ..., C args := t] declarations to behave as
expected, not introducing the [forall ...] variables to avoid unnecessary eta-expansions. Force to use { } in instance declarations when the class is a record even if it's a singleton. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12524 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/MSets/MSetList.v')
-rw-r--r--theories/MSets/MSetList.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/MSets/MSetList.v b/theories/MSets/MSetList.v
index b7b9a024a..c5e300cdd 100644
--- a/theories/MSets/MSetList.v
+++ b/theories/MSets/MSetList.v
@@ -225,7 +225,7 @@ Module MakeRaw (X: OrderedType) <: RawSets X.
Hint Resolve @ok.
Hint Constructors Ok.
- Instance Sort_Ok s `(Hs : Sort s) : Ok s := Hs.
+ Instance Sort_Ok s `(Hs : Sort s) : Ok s := { ok := Hs }.
Ltac inv_ok := match goal with
| H:Ok (_ :: _) |- _ => apply @ok in H; inversion_clear H; inv_ok