aboutsummaryrefslogtreecommitdiffhomepage
path: root/coq/ex/test-cases/multiple-files-multiple-dir/b
diff options
context:
space:
mode:
authorGravatar Hendrik Tews <hendrik@askra.de>2011-01-14 21:59:26 +0000
committerGravatar Hendrik Tews <hendrik@askra.de>2011-01-14 21:59:26 +0000
commite1f5de972cbc0eb8d88675366c34ee66aca1b1b4 (patch)
treea53834d26af2a1594b1289bd3d3c884e484f5780 /coq/ex/test-cases/multiple-files-multiple-dir/b
parent462d8403fbe048aac215d809bfa72e7360384071 (diff)
- more coq test cases (some with surprising and embarrassing bugs)
Diffstat (limited to 'coq/ex/test-cases/multiple-files-multiple-dir/b')
-rw-r--r--coq/ex/test-cases/multiple-files-multiple-dir/b/b1.v9
-rw-r--r--coq/ex/test-cases/multiple-files-multiple-dir/b/b2.v9
2 files changed, 18 insertions, 0 deletions
diff --git a/coq/ex/test-cases/multiple-files-multiple-dir/b/b1.v b/coq/ex/test-cases/multiple-files-multiple-dir/b/b1.v
new file mode 100644
index 00000000..afcd3941
--- /dev/null
+++ b/coq/ex/test-cases/multiple-files-multiple-dir/b/b1.v
@@ -0,0 +1,9 @@
+(* this file depends on ../a/a.v *)
+
+Definition a := 1.
+
+Require a.
+
+(*** Local Variables: ***)
+(*** coq-load-path: ("../a") ***)
+(*** End: ***)
diff --git a/coq/ex/test-cases/multiple-files-multiple-dir/b/b2.v b/coq/ex/test-cases/multiple-files-multiple-dir/b/b2.v
new file mode 100644
index 00000000..6d79572a
--- /dev/null
+++ b/coq/ex/test-cases/multiple-files-multiple-dir/b/b2.v
@@ -0,0 +1,9 @@
+(* this file depends on b1 and therefore indirectly on ../a/a.v *)
+
+Definition a := 2.
+
+Require b1.
+
+(*** Local Variables: ***)
+(*** coq-load-path: ("../a") ***)
+(*** End: ***)