aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/primitiveproj.v
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <mattam@mattam.org>2015-07-22 17:26:49 +0200
committerGravatar Matthieu Sozeau <mattam@mattam.org>2015-07-22 17:26:49 +0200
commit754775e39b5fa0342a1f4a46cbce0fc98d569d9d (patch)
treed907f1303514d557b901f949d5b02cc165a9992d /test-suite/success/primitiveproj.v
parentc07a9f1e558ab55de3011cbfc9749391ed60c768 (diff)
Extraction: fix primitive projection extraction.
Use expand projection to come back to the projection-as-constant encoding, dealing with parameters correctly.
Diffstat (limited to 'test-suite/success/primitiveproj.v')
-rw-r--r--test-suite/success/primitiveproj.v7
1 files changed, 7 insertions, 0 deletions
diff --git a/test-suite/success/primitiveproj.v b/test-suite/success/primitiveproj.v
index 068f8ac3c..125615c53 100644
--- a/test-suite/success/primitiveproj.v
+++ b/test-suite/success/primitiveproj.v
@@ -188,3 +188,10 @@ Set Printing All.
Check (@p' nat).
Check p'.
Unset Printing All.
+
+Record wrap (A : Type) := { unwrap : A; unwrap2 : A }.
+
+Definition term (x : wrap nat) := x.(unwrap).
+Definition term' (x : wrap nat) := let f := (@unwrap2 nat) in f x.
+Recursive Extraction term term'.
+(*Unset Printing Primitive Projection Parameters.*) \ No newline at end of file