summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/2464.v
blob: af7085872009577cdc66b5fdc97d037681821f1c (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
22
23
24
25
26
27
28
29
30
31
32
33
34
35
36
37
38
39
Require Import FSetWeakList.
Require Import FSetDecide.

Parameter Name : Set.
Axiom eq_Name_dec : forall (n : Name) (o : Name), {n = o} + {n <> o}.

Module DecidableName.
Definition t := Name.
Definition eq := @eq Name.
Definition eq_refl := @refl_equal Name.
Definition eq_sym := @sym_eq Name.
Definition eq_trans := @trans_eq Name.
Definition eq_dec := eq_Name_dec.
End DecidableName.

Module NameSetMod := Make(DecidableName).

Module NameSetDec := WDecide (NameSetMod).

Class PartPatchUniverse (pu_type1 pu_type2 : Type)
                       : Type := mkPartPatchUniverse {
}.
Class PatchUniverse {pu_type : Type}
                    (ppu : PartPatchUniverse pu_type pu_type)
                  : Type := mkPatchUniverse {
    pu_nameOf : pu_type -> Name
}.

Lemma foo : forall (pu_type : Type)
                   (ppu : PartPatchUniverse pu_type pu_type)
                   (patchUniverse : PatchUniverse ppu)
                   (ns ns1 ns2 : NameSetMod.t)
                   (containsOK : NameSetMod.Equal ns1 ns2)
                   (p : pu_type)
                   (HX1 : NameSetMod.Equal ns1 (NameSetMod.add (pu_nameOf p) ns)),
            NameSetMod.Equal ns2 (NameSetMod.add (pu_nameOf p) ns).
Proof.
NameSetDec.fsetdec.
Qed.