aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success
diff options
context:
space:
mode:
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.
+
+*)