aboutsummaryrefslogtreecommitdiffhomepage
path: root/coq/ex/test-cases/multiple-files-single-dir/f.v
blob: d36ccef6299981fc706493d2e3ae4661103ed8c8 (plain)
1
2
3
4
5
6
7
(* this file depends on d.v and e.v and therefore 
 * indirectly also on a.v, b.v and c.v
 *)

Require Import d e.

Definition a := 5.