aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2017-07-27 22:46:58 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2017-07-27 22:53:10 +0200
commit630f565077fa8f9ce9fdd0535b61901c6c539e02 (patch)
treec05020024afbd4520ab5b767b7421f7203a5c245 /test-suite
parent2a7ba998bf7d2c461fdbd8b710b7124395bafaa2 (diff)
Fixing bug #5671 (specialize unclean wrt Metas).
Diffstat (limited to 'test-suite')
-rw-r--r--test-suite/bugs/closed/5671.v7
1 files changed, 7 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/5671.v b/test-suite/bugs/closed/5671.v
new file mode 100644
index 000000000..c9a085045
--- /dev/null
+++ b/test-suite/bugs/closed/5671.v
@@ -0,0 +1,7 @@
+(* Fixing Meta-unclean specialize *)
+
+Require Import Setoid.
+Axiom a : forall x, x=0 -> True.
+Lemma lem (x y1 y2:nat) (H:x=0) (H0:eq y1 y2) : y1 = y2.
+specialize a with (1:=H). clear H x. intros _.
+setoid_rewrite H0.