aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/Inductive.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2013-05-08 17:44:00 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2013-05-08 17:44:00 +0000
commit0395451fb326551474a96ee802185070f4bf3595 (patch)
treedb741fd07023d2b6d0be372e47ee7ce13c8270d0 /test-suite/success/Inductive.v
parent3a569247c5d9260e89ed5a4230468cb60f6f53a0 (diff)
Moved isolated test params_ind.v to Inductive.v.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@16485 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite/success/Inductive.v')
-rw-r--r--test-suite/success/Inductive.v6
1 files changed, 6 insertions, 0 deletions
diff --git a/test-suite/success/Inductive.v b/test-suite/success/Inductive.v
index 5e59930f3..a63c99ebf 100644
--- a/test-suite/success/Inductive.v
+++ b/test-suite/success/Inductive.v
@@ -107,3 +107,9 @@ Set Implicit Arguments.
Inductive I A : A->Prop := C a : (forall A, A) -> I a.
*)
+
+(* Test recursively non-uniform parameters (was formerly in params_ind.v) *)
+
+Inductive list (A : Set) : Set :=
+ | nil : list A
+ | cons : A -> list (A -> A) -> list A.