summaryrefslogtreecommitdiff
path: root/test-suite/misc/deps/B/B.v
blob: f3cda70a9dcd07e624029e9bfa818900302f55d3 (plain)
1
2
3
4
5
6
7
Require A.

Definition c := A.b.
Lemma foo : c = false.
Proof.
reflexivity.
Qed.