From b1c0584f24cb3732e1704a85452f4fe535e50f33 Mon Sep 17 00:00:00 2001 From: Matthieu Sozeau Date: Fri, 9 May 2014 11:59:24 +0200 Subject: Restore implicit arguments of irreflexivity (fixes bug #3305). --- theories/Structures/OrderedType.v | 2 +- 1 file changed, 1 insertion(+), 1 deletion(-) (limited to 'theories/Structures/OrderedType.v') 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. -- cgit v1.2.3