aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/3664.v
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2014-09-27 20:40:26 +0200
committerGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2014-09-27 20:43:03 +0200
commit92a183f4ada641c0ab73dd0479e98df36eeeb365 (patch)
tree3aa4634fbb5fb6253f0aeba7fd505c453ce402c9 /test-suite/bugs/closed/3664.v
parent3ca949d4069308cf71c8f22b8dfc89e95a3834c1 (diff)
Fix bug #3664 by refolding projections that don't reduce in cbn.
Diffstat (limited to 'test-suite/bugs/closed/3664.v')
-rw-r--r--test-suite/bugs/closed/3664.v23
1 files changed, 23 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/3664.v b/test-suite/bugs/closed/3664.v
new file mode 100644
index 000000000..41de74ff3
--- /dev/null
+++ b/test-suite/bugs/closed/3664.v
@@ -0,0 +1,23 @@
+Module NonPrim.
+ Unset Primitive Projections.
+ Record c := { d : Set }.
+ Definition a x := d x.
+ Goal forall x, a x.
+ intro x.
+ Fail progress simpl. (* [progress simpl] fails correctly *)
+ Fail progress cbn. (* [progress cbn] fails correctly *)
+ admit.
+ Defined.
+End NonPrim.
+
+Module Prim.
+ Set Primitive Projections.
+ Record c := { d : Set }.
+ Definition a x := d x.
+ Goal forall x, a x.
+ intro x.
+ Fail progress simpl. (* [progress simpl] fails correctly *)
+ Fail progress cbn. (* [cbn] succeeds incorrectly, giving [d x] *)
+ admit.
+ Defined.
+End Prim. \ No newline at end of file