summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/3798.v
diff options
context:
space:
mode:
Diffstat (limited to 'test-suite/bugs/closed/3798.v')
-rw-r--r--test-suite/bugs/closed/3798.v12
1 files changed, 12 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/3798.v b/test-suite/bugs/closed/3798.v
new file mode 100644
index 00000000..b9f0daa7
--- /dev/null
+++ b/test-suite/bugs/closed/3798.v
@@ -0,0 +1,12 @@
+Require Import TestSuite.admit.
+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.