aboutsummaryrefslogtreecommitdiff
path: root/test-suite
diff options
context:
space:
mode:
authorGaëtan Gilbert2018-12-19 12:43:23 +0100
committerGaëtan Gilbert2018-12-19 12:43:23 +0100
commitd3d142f406239b6e528d27454d1b3f4e3d6fd4ea (patch)
tree698fa2735529982d7a10ccaf711b554d0262d0db /test-suite
parent2cad4dec40cef2aecb19c5a0e5a1368392be8d88 (diff)
coqchk: fix check for kelim with functors
Diffstat (limited to 'test-suite')
-rw-r--r--test-suite/coqchk/inductive_functor_squash.v15
1 files changed, 15 insertions, 0 deletions
diff --git a/test-suite/coqchk/inductive_functor_squash.v b/test-suite/coqchk/inductive_functor_squash.v
new file mode 100644
index 0000000000..9d33fafc4c
--- /dev/null
+++ b/test-suite/coqchk/inductive_functor_squash.v
@@ -0,0 +1,15 @@
+
+
+Module Type T.
+ Parameter f : nat -> Type.
+End T.
+
+Module F(A:T).
+ Inductive ind : Prop :=
+ C : A.f 0 -> ind.
+End F.
+
+Module A. Definition f (x:nat) := True. End A.
+
+Module M := F A.
+(* M.ind could eliminate into Set/Type even though F.ind can't *)