aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/3596.v
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2014-09-11 11:21:38 +0200
committerGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2014-09-11 13:30:33 +0200
commit12ef55e112a1ccfe00c8880e0ba5958e02ab97e1 (patch)
treece90736b1e1b1032884d8cee832f808553d27d70 /test-suite/bugs/closed/3596.v
parent6e2b4a66b9f176555eb541cbee762d3cf3fc183c (diff)
Fix bug #3596, wrong treatment of projections in compute_constelim_direct.
Diffstat (limited to 'test-suite/bugs/closed/3596.v')
-rw-r--r--test-suite/bugs/closed/3596.v18
1 files changed, 18 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/3596.v b/test-suite/bugs/closed/3596.v
new file mode 100644
index 000000000..d6c1c949d
--- /dev/null
+++ b/test-suite/bugs/closed/3596.v
@@ -0,0 +1,18 @@
+Set Implicit Arguments.
+Record foo := { fx : nat }.
+Set Primitive Projections.
+Record bar := { bx : nat }.
+Definition Foo (f : foo) : f = f.
+ destruct f as [fx]; destruct fx; admit.
+Defined.
+Definition Bar (b : bar) : b = b.
+ destruct b as [fx]; destruct fx; admit.
+Defined.
+Goal forall f b, Bar b = Bar b -> Foo f = Foo f.
+ intros f b.
+ destruct f, b.
+ simpl.
+ Fail progress unfold Bar. (* success *)
+ Fail progress unfold Foo. (* failed to progress *)
+ reflexivity.
+Qed. \ No newline at end of file