aboutsummaryrefslogtreecommitdiff
diff options
context:
space:
mode:
authorEnrico Tassi2019-02-22 14:10:18 +0100
committerEnrico Tassi2019-02-25 14:12:10 +0100
commit565cefdb051339a601b9977e163ee4ffbba75274 (patch)
treea8c10b0f1f999f8d8547f887606815bdc6857cfa
parent8cad12e0e48eae83773667c2fab7d2570ed43ed2 (diff)
add testcase for primitive projection
-rw-r--r--test-suite/bugs/closed/bug_9598.v13
1 files changed, 13 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/bug_9598.v b/test-suite/bugs/closed/bug_9598.v
index daf4d3f847..00bbfcf5d9 100644
--- a/test-suite/bugs/closed/bug_9598.v
+++ b/test-suite/bugs/closed/bug_9598.v
@@ -21,3 +21,16 @@ Module fixpoint.
Fixpoint rec_ko (x : nat) : nat := fst (alias_K 0 (rec_ko x)).
End fixpoint.
+
+Module primproj.
+
+ Set Primitive Projections.
+
+ Inductive pair := K { fst : nat; snd : nat }.
+
+ Definition alias_K a b := K a b.
+
+ Fixpoint rec (x : nat) : nat := fst (K 0 (rec x)).
+ Fixpoint rec_ko (x : nat) : nat := fst (alias_K 0 (rec_ko x)).
+
+End primproj.