aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/output/Inductive.v
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2017-09-23 12:25:35 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2017-12-14 15:57:51 +0100
commit63d582c6cd12bc3f8134a5aa9e3bdbca0dd2e9ca (patch)
tree368bc9298c9694c705bb66d89638a96f54aa8a89 /test-suite/output/Inductive.v
parente0c06c7dac30b9959a3eb90b0c1d324f061a8660 (diff)
Fixing a bug of Print for inductive types with let-ins in parameters.
Adding a "let-in"-sensitive function hnf_prod_applist_assum to instantiate parameters and using it for printing. Thanks to PMP for reporting.
Diffstat (limited to 'test-suite/output/Inductive.v')
-rw-r--r--test-suite/output/Inductive.v4
1 files changed, 4 insertions, 0 deletions
diff --git a/test-suite/output/Inductive.v b/test-suite/output/Inductive.v
index 8db8956e3..8ff91268a 100644
--- a/test-suite/output/Inductive.v
+++ b/test-suite/output/Inductive.v
@@ -1,3 +1,7 @@
Fail Inductive list' (A:Set) : Set :=
| nil' : list' A
| cons' : A -> list' A -> list' (A*A).
+
+(* Check printing of let-ins *)
+Inductive foo (A : Type) (x : A) (y := x) := Foo.
+Print foo.