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/MSets/MSetInterface.v | 2 +- 1 file changed, 1 insertion(+), 1 deletion(-) (limited to 'theories/MSets') 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. -- cgit v1.2.3