summaryrefslogtreecommitdiff
path: root/test-suite/misc/deps/client/bar.v
blob: 6296941862def75639e5a300269e666321646730 (plain)
1
2
3
4
5
6
7
8
9
10
11
(* We assume the file compiled with -R ../lib lib -R . client *)
(* foo alone should refer to client.foo because -R . client comes last *)

Require Import foo.
Goal a = 1.
reflexivity.
Qed.
Require Import lib.foo.
Goal a = 0.
reflexivity.
Qed.