diff options
author | Matthieu Sozeau <mattam@mattam.org> | 2014-05-09 11:59:24 +0200 |
---|---|---|
committer | Matthieu Sozeau <mattam@mattam.org> | 2014-05-09 11:59:24 +0200 |
commit | b1c0584f24cb3732e1704a85452f4fe535e50f33 (patch) | |
tree | 1e5285441beb5567c44cda5ee99ec4fd9a6ac140 /theories/Structures | |
parent | a8ee1bef887fbf14ffe1380152993b0db4298c98 (diff) |
Restore implicit arguments of irreflexivity (fixes bug #3305).
Diffstat (limited to 'theories/Structures')
-rw-r--r-- | theories/Structures/OrderedType.v | 2 |
1 files changed, 1 insertions, 1 deletions
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. |