aboutsummaryrefslogtreecommitdiff
diff options
context:
space:
mode:
authorPierre-Marie Pédrot2015-01-24 10:34:26 +0100
committerPierre-Marie Pédrot2015-01-25 12:49:12 +0100
commitd3934986fb2ff0d563a1a2a89ba5fbbefb53f0fd (patch)
treed839cbde3d3973ec3814f233b187d41db92c6889
parent27aec3933031ec5e87738965c25ffa51863c9400 (diff)
Test for bug #3798.
-rw-r--r--test-suite/bugs/closed/3798.v11
1 files changed, 11 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/3798.v b/test-suite/bugs/closed/3798.v
new file mode 100644
index 0000000000..623822e990
--- /dev/null
+++ b/test-suite/bugs/closed/3798.v
@@ -0,0 +1,11 @@
+Require Setoid.
+
+Parameter f : nat -> nat.
+Axiom a : forall n, 0 < n -> f n = 0.
+Hint Rewrite a using ( simpl; admit ).
+
+Goal f 1 = 0.
+Proof.
+ rewrite_strat (topdown (hints core)).
+ reflexivity.
+Qed.