aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/MSets/MSetAVL.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/MSetAVL.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/MSetAVL.v')
-rw-r--r--theories/MSets/MSetAVL.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/theories/MSets/MSetAVL.v b/theories/MSets/MSetAVL.v
index 8f825c584..56186e623 100644
--- a/theories/MSets/MSetAVL.v
+++ b/theories/MSets/MSetAVL.v
@@ -538,7 +538,7 @@ Definition IsOk := bst.
Class Ok (s:t) : Prop := { ok : bst s }.
-Instance bst_Ok s (Hs : bst s) : Ok s := Hs.
+Instance bst_Ok s (Hs : bst s) : Ok s := { ok := Hs }.
Fixpoint ltb_tree x s :=
match s with
@@ -1523,7 +1523,7 @@ Proof.
destruct (andb_prop _ _ H0); auto.
(* <- *)
induction s; simpl; auto.
- intros.
+ intros. red in H0.
rewrite IHs1; try red; auto.
rewrite IHs2; try red; auto.
generalize (H0 t0).