diff options
| author | letouzey | 2013-03-25 12:22:56 +0000 |
|---|---|---|
| committer | letouzey | 2013-03-25 12:22:56 +0000 |
| commit | b37bb277285db6b35ab4d147dddf3e45ae9707d3 (patch) | |
| tree | 1e0b0972fdd0fe48b4f809295ed99edc91cb0178 | |
| parent | 52c3aea2d3a9e03c307166ec667bc7ad90ae4fed (diff) | |
Add the test-case of bug 2750 in the test-suite
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@16362 85f007b7-540e-0410-9357-904b9bb8a0f7
| -rw-r--r-- | test-suite/bugs/closed/shouldsucceed/2750.v | 23 |
1 files changed, 23 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/shouldsucceed/2750.v b/test-suite/bugs/closed/shouldsucceed/2750.v new file mode 100644 index 0000000000..fc580f1018 --- /dev/null +++ b/test-suite/bugs/closed/shouldsucceed/2750.v @@ -0,0 +1,23 @@ + +Module Type ModWithRecord. + + Record foo : Type := + { A : nat + ; B : nat + }. +End ModWithRecord. + +Module Test_ModWithRecord (M : ModWithRecord). + + Definition test1 : M.foo := + {| M.A := 0 + ; M.B := 2 + |}. + + Module B := M. + + Definition test2 : M.foo := + {| M.A := 0 + ; M.B := 2 + |}. +End Test_ModWithRecord.
\ No newline at end of file |
