diff options
author | barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2010-03-12 15:30:51 +0000 |
---|---|---|
committer | barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2010-03-12 15:30:51 +0000 |
commit | 74db2b0098893a5912d7480a259ad91664a86120 (patch) | |
tree | bf9c4fdff014b335c46684ffd211ce496a6f947c /test-suite/success | |
parent | dba2ae9fa1eb01d795d36b209aee6045967ba00a (diff) |
fixed confusion between number of cstr arguments and number of pattern variables (which include let-ins in cstr type)
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12864 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite/success')
-rw-r--r-- | test-suite/success/Inductive.v | 9 |
1 files changed, 9 insertions, 0 deletions
diff --git a/test-suite/success/Inductive.v b/test-suite/success/Inductive.v index 203fbbb77..8ffe4fcdb 100644 --- a/test-suite/success/Inductive.v +++ b/test-suite/success/Inductive.v @@ -54,6 +54,15 @@ Check | Build_B x0 x1 => f x0 x1 end). +(* Check inductive types with local definitions (constructors) *) + +Inductive I1 : Set := c (_:I1) (_:=0). + +Check (fun x:I1 => + match x with + | c i n => (i,n) + end). + (* Check implicit parameters of inductive types (submitted by Pierre Casteran and also implicit in #338) *) |