aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/MSets/MSetInterface.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/MSetInterface.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/MSetInterface.v')
-rw-r--r--theories/MSets/MSetInterface.v10
1 files changed, 1 insertions, 9 deletions
diff --git a/theories/MSets/MSetInterface.v b/theories/MSets/MSetInterface.v
index 0de28d5e8..ae26fa7ed 100644
--- a/theories/MSets/MSetInterface.v
+++ b/theories/MSets/MSetInterface.v
@@ -340,7 +340,7 @@ Module Type WRawSets (E : DecidableType).
(** Is a set well-formed or ill-formed ? *)
Parameter IsOk : t -> Prop.
- Class Ok (s:t) : Prop := { ok : IsOk s }.
+ Class Ok (s:t) : Prop := ok : IsOk s.
(** In order to be able to validate (at least some) particular sets as
well-formed, we ask for a boolean function for (semi-)deciding
@@ -425,14 +425,6 @@ Module Type WRawSets (E : DecidableType).
End Spec.
-(*
- BUG ?! When the Instance *_ok were under a section,
- this re-export was mandatory !! BUG in Global Instance ?
- Hint Resolve empty_ok add_ok remove_ok union_ok inter_ok
- diff_ok singleton_ok filter_ok partition_ok1 partition_ok2
- : typeclass_instances.
-*)
-
End WRawSets.
(** From weak raw sets to weak usual sets *)