From 867a119264666100ec7f6fd5d080a2f8cd8124fb Mon Sep 17 00:00:00 2001 From: letouzey Date: Sun, 14 May 2006 09:07:17 +0000 Subject: reparartion d'un petit oubli cassant PrecedenceGraph git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@8815 85f007b7-540e-0410-9357-904b9bb8a0f7 --- theories/FSets/FSetProperties.v | 2 +- 1 file changed, 1 insertion(+), 1 deletion(-) (limited to 'theories') diff --git a/theories/FSets/FSetProperties.v b/theories/FSets/FSetProperties.v index 44abc0f1b..8a5156e1c 100644 --- a/theories/FSets/FSetProperties.v +++ b/theories/FSets/FSetProperties.v @@ -21,7 +21,7 @@ Require Import FSetFacts. Set Implicit Arguments. Unset Strict Implicit. -Hint Unfold transpose compat_op. +Hint Unfold transpose compat_op compat_nat. Hint Extern 1 (Setoid_Theory _ _) => constructor; congruence. Module Properties (M: S). -- cgit v1.2.3