aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/MSets/MSetList.v
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-01-12 16:54:08 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-01-12 16:54:08 +0000
commit8bfc7b2ac5a4d6d218071611a5002e513e731451 (patch)
tree424b2ea522c86f5ab2d156821e625812231df751 /theories/MSets/MSetList.v
parentb264811fbed75caff5deb2b6eb78a327dc134f68 (diff)
MSets: Class Ok becomes a definition instead of an inductive (thanks Matthieu)
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12656 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/MSets/MSetList.v')
-rw-r--r--theories/MSets/MSetList.v10
1 files changed, 5 insertions, 5 deletions
diff --git a/theories/MSets/MSetList.v b/theories/MSets/MSetList.v
index b0caf6692..c29742332 100644
--- a/theories/MSets/MSetList.v
+++ b/theories/MSets/MSetList.v
@@ -225,17 +225,17 @@ Module MakeRaw (X: OrderedType) <: RawSets X.
Definition IsOk := Sort.
- Class Ok (s:t) : Prop := { ok : Sort s }.
+ Class Ok (s:t) : Prop := ok : Sort s.
Hint Resolve @ok.
- Hint Constructors Ok.
+ Hint Unfold Ok.
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
+ | H:Ok (_ :: _) |- _ => inversion_clear H; inv_ok
| H:Ok nil |- _ => clear H; inv_ok
- | H:Sort ?l |- _ => generalize (Build_Ok H); clear H; intro H; inv_ok
+ | H:Sort ?l |- _ => change (Ok l) in H; inv_ok
| _ => idtac
end.
@@ -439,7 +439,7 @@ Module MakeRaw (X: OrderedType) <: RawSets X.
Global Instance diff_ok s s' `(Ok s, Ok s') : Ok (diff s s').
Proof.
- induction2. constructors; auto. apply @ok; auto.
+ induction2. constructors; auto.
Qed.
Lemma diff_spec :