aboutsummaryrefslogtreecommitdiffhomepage
path: root/coq/ex/test-cases/multiple-files-multiple-dir/b/b1.v
blob: afcd3941199adcd24b7e8192f4b1a0eacdc45635 (plain)
1
2
3
4
5
6
7
8
9
(* this file depends on ../a/a.v *)

Definition a := 1.

Require a.

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