aboutsummaryrefslogtreecommitdiffhomepage
path: root/coq/ex/test-cases/multiple-files-multiple-dir/c/c.v
blob: 5171340ce3b9365270734ee5c144737ecbe566ac (plain)
1
2
3
4
5
6
7
8
9
10
11
(* this file depends on ../b/b2 and therefore indirectly 
 * on ../b/b1 and ../a/a.v 
 *)

Definition a := 2.

Require b2.

(*** Local Variables: ***)
(*** coq-load-path: ("../a" "../b") ***)
(*** End: ***)