aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-01-12 11:04:23 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-01-12 11:04:23 +0000
commitcbb46eafff8a1225ebef2f790b8854516f310d09 (patch)
treee31e3d1aad028de201148d2d78508b0bcc91793a /test-suite/success
parent1a9feee3ab72de653533effafd6365648b3d7970 (diff)
Temporary fix to compensate the loss of descent on dependent
conjunctions (defined records now supported again but not unregistered ones). git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12650 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite/success')
-rw-r--r--test-suite/success/apply.v17
1 files changed, 17 insertions, 0 deletions
diff --git a/test-suite/success/apply.v b/test-suite/success/apply.v
index 3fc8a9792..cb55432fb 100644
--- a/test-suite/success/apply.v
+++ b/test-suite/success/apply.v
@@ -348,3 +348,20 @@ Goal True.
eapply (fun (A:Prop) (x:A) => conj I x).
exact I.
Qed.
+
+(* The following was not accepted from r12612 to r12649 *)
+
+Record sig0 := { p1 : nat; p2 : p1 = 0 }.
+
+Goal forall x : sig0, p1 x = 0.
+intro x;
+apply x.
+Qed.
+
+(* The following was accepted before r12612 but is still not accepted in r12650
+
+Goal forall x : { x:nat | x = 0}, proj1_sig x = 0.
+intro x;
+apply x.
+
+*)