aboutsummaryrefslogtreecommitdiffhomepage
path: root/coq/ex/test-cases/multiple-files-single-dir/d.v
blob: b0c47e8b30041ea7ad4c78d9786ddb4a889482a7 (plain)
1
2
3
4
5
(* this file depends on a.v and b.v *)

Require Import a b.

Definition a := 3.