aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
-rw-r--r--theories/Classes/RelationClasses.v2
-rw-r--r--theories/MSets/MSetInterface.v2
-rw-r--r--theories/Structures/OrderedType.v2
3 files changed, 4 insertions, 2 deletions
diff --git a/theories/Classes/RelationClasses.v b/theories/Classes/RelationClasses.v
index 61edb2b98..3bd9dcd12 100644
--- a/theories/Classes/RelationClasses.v
+++ b/theories/Classes/RelationClasses.v
@@ -202,6 +202,8 @@ Hint Extern 3 (PreOrder (flip _)) => class_apply flip_PreOrder : typeclass_insta
Hint Extern 4 (subrelation (flip _) _) =>
class_apply @subrelation_symmetric : typeclass_instances.
+Arguments irreflexivity {A R Irreflexive} [x] _.
+
Hint Resolve irreflexivity : ord.
Unset Implicit Arguments.
diff --git a/theories/MSets/MSetInterface.v b/theories/MSets/MSetInterface.v
index a61ef8bcd..bd8811689 100644
--- a/theories/MSets/MSetInterface.v
+++ b/theories/MSets/MSetInterface.v
@@ -595,7 +595,7 @@ Module Raw2SetsOn (O:OrderedType)(M:RawSets O) <: SetsOn O.
(** Specification of [lt] *)
Instance lt_strorder : StrictOrder lt.
Proof. constructor ; unfold lt; red.
- unfold complement. red. intros. apply (irreflexivity _ H).
+ unfold complement. red. intros. apply (irreflexivity H).
intros. transitivity y; auto.
Qed.
diff --git a/theories/Structures/OrderedType.v b/theories/Structures/OrderedType.v
index fb28e0cfc..fa08f9366 100644
--- a/theories/Structures/OrderedType.v
+++ b/theories/Structures/OrderedType.v
@@ -328,7 +328,7 @@ Module KeyOrderedType(O:OrderedType).
Proof. split; eauto. Qed.
Global Instance ltk_strorder : StrictOrder ltk.
- Proof. constructor; eauto. intros x; apply (irreflexivity (fst x)). Qed.
+ Proof. constructor; eauto. intros x; apply (irreflexivity (x:=fst x)). Qed.
Global Instance ltk_compat : Proper (eqk==>eqk==>iff) ltk.
Proof.