aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/setoid_test.v
diff options
context:
space:
mode:
authorGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2013-06-10 15:42:03 +0000
committerGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2013-06-10 15:42:03 +0000
commitf97121161c9e6c11eea4ad8c4303d0bd083c6672 (patch)
tree692691d69da481545f3501402c58de1ba18545b3 /test-suite/success/setoid_test.v
parent7309e19cad53a3e07aa4db6245a91b56cf3fc03b (diff)
Fix [setoid_rewrite] forgetting some evars that are produced when typechecking a lemma
to apply, fixes test-suite test. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@16569 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite/success/setoid_test.v')
-rw-r--r--test-suite/success/setoid_test.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/test-suite/success/setoid_test.v b/test-suite/success/setoid_test.v
index 653b5bf9a..be0d49e00 100644
--- a/test-suite/success/setoid_test.v
+++ b/test-suite/success/setoid_test.v
@@ -153,7 +153,7 @@ End mult.
does not fix the instance at the first unification, use [at], or simply rewrite for
this semantics. *)
-Require Import Arith.
+Parameter beq_nat : forall x y : nat, bool.
Class Foo (A : Type) := {foo_neg : A -> A ; foo_prf : forall x : A, x = foo_neg x}.
Instance: Foo nat. admit. Defined.