From a22219b5eec49a731921fda7e5f8711b45725531 Mon Sep 17 00:00:00 2001 From: msozeau Date: Mon, 8 Jun 2009 17:24:53 +0000 Subject: Do a fixpoint on the result of typeclass search to force the resolution of generated evars, not doing any backtracking yet. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12175 85f007b7-540e-0410-9357-904b9bb8a0f7 --- theories/Classes/Morphisms.v | 2 +- 1 file changed, 1 insertion(+), 1 deletion(-) (limited to 'theories/Classes/Morphisms.v') diff --git a/theories/Classes/Morphisms.v b/theories/Classes/Morphisms.v index 9e1eecd1d..595ad1297 100644 --- a/theories/Classes/Morphisms.v +++ b/theories/Classes/Morphisms.v @@ -325,7 +325,7 @@ Proof. firstorder. Qed. Lemma proper_proper_proxy `(Proper A R x) : ProperProxy R x. Proof. firstorder. Qed. -Hint Extern 1 (ProperProxy _ _) => class_apply eq_proper_proxy || class_apply @reflexive_proper_proxy : typeclass_instances. +Hint Extern 1 (ProperProxy _ _) => class_apply @eq_proper_proxy || class_apply @reflexive_proper_proxy : typeclass_instances. Hint Extern 2 (ProperProxy ?R _) => not_evar R ; class_apply @proper_proper_proxy : typeclass_instances. (** [R] is Reflexive, hence we can build the needed proof. *) -- cgit v1.2.3