summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/3938.v
diff options
context:
space:
mode:
Diffstat (limited to 'test-suite/bugs/closed/3938.v')
-rw-r--r--test-suite/bugs/closed/3938.v8
1 files changed, 8 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/3938.v b/test-suite/bugs/closed/3938.v
new file mode 100644
index 00000000..859e9f01
--- /dev/null
+++ b/test-suite/bugs/closed/3938.v
@@ -0,0 +1,8 @@
+Require Import TestSuite.admit.
+Require Import Coq.Arith.PeanoNat.
+Hint Extern 1 => admit : typeclass_instances.
+Require Import Setoid.
+Goal forall a b (f : nat -> Set) (R : nat -> nat -> Prop),
+ Equivalence R -> R a b -> f a = f b.
+ intros a b f H.
+ intros. Fail rewrite H1.