summaryrefslogtreecommitdiff
path: root/test-suite/output/qualification.v
blob: d39097e2dddc5f92bb93ec3a859c001306603566 (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
Module Type T1.
  Parameter t : Type.
End T1.

Module Type T2.
  Declare Module M : T1.
  Parameter t : Type.
  Parameter test : t = M.t.
End T2.

Module M1 <: T1.
  Definition t : Type := bool.
End M1.

Module M2 <: T2.
  Module M := M1.
  Definition t : Type := nat.
  Lemma test : t = t. Proof. reflexivity. Qed.
End M2.