summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/4078.v
blob: 236cd2fbb1df9051f7c42ef723853bb42a057e5b (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
Module Type S.

Axiom foo : nat.

End S.

Module M : S.

Definition bar := 0.
Definition foo := bar.

End M.

Print All Dependencies M.foo.