aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/MSets
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <mattam@mattam.org>2014-05-09 11:59:24 +0200
committerGravatar Matthieu Sozeau <mattam@mattam.org>2014-05-09 11:59:24 +0200
commitb1c0584f24cb3732e1704a85452f4fe535e50f33 (patch)
tree1e5285441beb5567c44cda5ee99ec4fd9a6ac140 /theories/MSets
parenta8ee1bef887fbf14ffe1380152993b0db4298c98 (diff)
Restore implicit arguments of irreflexivity (fixes bug #3305).
Diffstat (limited to 'theories/MSets')
-rw-r--r--theories/MSets/MSetInterface.v2
1 files changed, 1 insertions, 1 deletions
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.