Skip to content

Commit 911dd7d

Browse files
authored
Merge pull request #906 from JasonGross/coq-8.16+remove-dead-quotation-code
Remove some duplicate code in quotation
2 parents 06da2d3 + e668975 commit 911dd7d

File tree

11 files changed

+15
-36
lines changed

11 files changed

+15
-36
lines changed

quotation/theories/ToTemplate/Coq/FSets.v

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1,5 +1,5 @@
11
From Coq Require Import Structures.Equalities Structures.OrdersAlt FMapInterface FMapList FMapAVL FMapFullAVL FMapFacts.
2-
From MetaCoq.Utils Require Import MCUtils.
2+
From MetaCoq.Utils Require Import MCUtils MCFSets.
33
From MetaCoq.Quotation.ToTemplate Require Import Init.
44
From MetaCoq.Quotation.ToTemplate Require Import (hints) Coq.Numbers Coq.Init Coq.Lists.
55
From MetaCoq.Quotation.ToTemplate.QuotationOf.Coq.Structures Require Import OrdersAlt.Sig.

quotation/theories/ToTemplate/Coq/MSets.v

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -1,4 +1,5 @@
11
From Coq Require Import MSetInterface MSetList MSetAVL MSetFacts MSetProperties MSetDecide.
2+
From MetaCoq.Utils Require Import MCMSets.
23
From MetaCoq.Quotation.ToTemplate Require Import Init.
34
From MetaCoq.Quotation.ToTemplate Require Import (hints) Coq.Numbers Coq.Init Coq.Lists.
45
From MetaCoq.Quotation.ToTemplate.QuotationOf.Coq.Structures Require Import Orders.Sig.

quotation/theories/ToTemplate/QuotationOf/Coq/FSets/FMapAVL/Sig.v

Lines changed: 2 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -1,15 +1,14 @@
11
From Coq.FSets Require Import FMapAVL.
22
From Coq.Structures Require Import Equalities OrdersAlt.
3+
From MetaCoq.Utils Require Import MCFSets.
34
From MetaCoq.Quotation.ToTemplate Require Import Init.
45
From MetaCoq.Quotation.ToTemplate.QuotationOf.Coq.Structures Require Import OrdersAlt.Sig.
56
From MetaCoq.Quotation.ToTemplate.QuotationOf.Coq.FSets Require Import FMapList.Sig.
67
Import List.ListNotations.
78
Local Open Scope list_scope.
89

910
Module FMapAVL.
10-
Module Type MakeSig (T : OrderedTypeOrig) := Nop <+ FMapAVL.Make T.
11-
12-
Module Type QuotationOfMake (T : OrderedTypeOrig) (M : MakeSig T).
11+
Module Type QuotationOfMake (T : OrderedTypeOrig) (M : FMapAVL.MakeSig T).
1312
Module qRaw.
1413
Module qProofs.
1514
Module qMX := Nop <+ QuotationOfOrderedTypeOrigFacts T M.Raw.Proofs.MX.

quotation/theories/ToTemplate/QuotationOf/Coq/FSets/FMapFacts/Sig.v

Lines changed: 1 addition & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -1,10 +1,9 @@
11
From Coq.FSets Require Import FMapFacts.
22
From Coq.Structures Require Import Orders.
3+
From MetaCoq.Utils Require Import MCFSets.
34
From MetaCoq.Quotation.ToTemplate Require Import Init.
45

56
Module Export FSets.
6-
Module Type WFacts_funSig (E : DecidableTypeOrig) (M : WSfun E) := Nop <+ WFacts_fun E M.
7-
87
Module Type QuotationOfWFacts_fun (E : DecidableTypeOrig) (M : WSfun E) (F : WFacts_funSig E M).
98
MetaCoq Run (tmDeclareQuotationOfModule everything (Some export) "F").
109
End QuotationOfWFacts_fun.

quotation/theories/ToTemplate/QuotationOf/Coq/FSets/FMapList/Sig.v

Lines changed: 2 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -1,14 +1,13 @@
11
From Coq.FSets Require Import FMapList.
22
From Coq.Structures Require Import Equalities OrdersAlt.
3+
From MetaCoq.Utils Require Import MCFSets.
34
From MetaCoq.Quotation.ToTemplate Require Import Init.
45
From MetaCoq.Quotation.ToTemplate.QuotationOf.Coq.Structures Require Import OrdersAlt.Sig.
56
Import List.ListNotations.
67
Local Open Scope list_scope.
78

89
Module FMapList.
9-
Module Type RawSig (T : OrderedTypeOrig) := Nop <+ FMapList.Raw T.
10-
11-
Module Type QuotationOfRaw (T : OrderedTypeOrig) (M : RawSig T).
10+
Module Type QuotationOfRaw (T : OrderedTypeOrig) (M : FMapList.RawSig T).
1211
Module qMX := Nop <+ QuotationOfOrderedTypeOrigFacts T M.MX.
1312
Module qPX := Nop <+ QuotationOfKeyOrderedTypeOrig T M.PX.
1413
Export (hints) qMX qPX.
Lines changed: 2 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -1,11 +1,10 @@
11
From Coq.Structures Require Import Orders.
22
From Coq.MSets Require Import MSetAVL.
3+
From MetaCoq.Utils Require Import MCMSets.
34
From MetaCoq.Quotation.ToTemplate Require Import Init.
45

56
Module MSetAVL.
6-
Module Type MakeSig (T : OrderedType) := Nop <+ MSetAVL.Make T.
7-
8-
Module Type QuotationOfMake (T : OrderedType) (M : MakeSig T).
7+
Module Type QuotationOfMake (T : OrderedType) (M : MSetAVL.MakeSig T).
98
MetaCoq Run (tmDeclareQuotationOfModule everything (Some export) "M").
109
End QuotationOfMake.
1110
End MSetAVL.

quotation/theories/ToTemplate/QuotationOf/Coq/MSets/MSetDecide/Sig.v

Lines changed: 1 addition & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -1,11 +1,8 @@
11
From Coq.MSets Require Import MSetInterface MSetDecide.
2+
From MetaCoq.Utils Require Import MCMSets.
23
From MetaCoq.Quotation.ToTemplate Require Import Init.
34

45
Module Export MSets.
5-
Module Type WDecideOnSig (E : DecidableType) (M : WSetsOn E) := Nop <+ WDecideOn E M.
6-
Module Type WDecideSig (M : WSets) := Nop <+ WDecide M.
7-
Module Type DecideSig (M : WSets) := Nop <+ Decide M.
8-
96
Module Type QuotationOfWDecideOn (E : DecidableType) (M : WSetsOn E) (F : WDecideOnSig E M).
107
MetaCoq Run (tmDeclareQuotationOfModule everything (Some export) "F").
118
End QuotationOfWDecideOn.

quotation/theories/ToTemplate/QuotationOf/Coq/MSets/MSetFacts/Sig.v

Lines changed: 1 addition & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -1,11 +1,8 @@
11
From Coq.MSets Require Import MSetFacts.
2+
From MetaCoq.Utils Require Import MCMSets.
23
From MetaCoq.Quotation.ToTemplate Require Import Init.
34

45
Module Export MSets.
5-
Module Type WFactsOnSig (E : DecidableType) (M : WSetsOn E) := Nop <+ WFactsOn E M.
6-
Module Type WFactsSig (M : WSets) := Nop <+ WFacts M.
7-
Module Type FactsSig (M : WSets) := Nop <+ Facts M.
8-
96
Module Type QuotationOfWFactsOn (E : DecidableType) (M : WSetsOn E) (F : WFactsOnSig E M).
107
MetaCoq Run (tmDeclareQuotationOfModule everything (Some export) "F").
118
End QuotationOfWFactsOn.

quotation/theories/ToTemplate/QuotationOf/Coq/MSets/MSetInterface/Sig.v

Lines changed: 0 additions & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -21,8 +21,3 @@ Module Type QuotationOfSetsOn (E : OrderedType) (Import M : SetsOn E).
2121
#[export] Declare Instance qchoose_spec3 : quotation_of M.choose_spec3.
2222
End QuotationOfSetsOn.
2323
Module Type QuotationOfSets (M : Sets) := QuotationOfSetsOn M.E M.
24-
25-
Module Type UsualSets <: Sets.
26-
Declare Module E : UsualOrderedType.
27-
Include SetsOn E.
28-
End UsualSets.

quotation/theories/ToTemplate/QuotationOf/Coq/MSets/MSetList/Sig.v

Lines changed: 3 additions & 6 deletions
Original file line numberDiff line numberDiff line change
@@ -1,5 +1,6 @@
11
From Coq.Structures Require Import Equalities Orders.
22
From Coq.MSets Require Import MSetList.
3+
From MetaCoq.Utils Require Import MCMSets.
34
From MetaCoq.Quotation.ToTemplate Require Import Init.
45
From MetaCoq.Quotation.ToTemplate.QuotationOf.Coq.MSets Require Import MSetInterface.Sig.
56

@@ -13,15 +14,11 @@ Module Type QuotationOfSWithLeibniz (S : SWithLeibniz).
1314
End QuotationOfSWithLeibniz.
1415

1516
Module MSetList.
16-
Module Type MakeSig (T : OrderedType) := Nop <+ MSetList.Make T.
17-
18-
Module Type QuotationOfMake (T : OrderedType) (M : MakeSig T).
17+
Module Type QuotationOfMake (T : OrderedType) (M : MSetList.MakeSig T).
1918
MetaCoq Run (tmDeclareQuotationOfModule everything (Some export) "M").
2019
End QuotationOfMake.
2120

22-
Module Type MakeWithLeibnizSig (X : OrderedTypeWithLeibniz) := Nop <+ MakeWithLeibniz X.
23-
24-
Module Type QuotationOfMakeWithLeibniz (T : OrderedTypeWithLeibniz) (M : MakeWithLeibnizSig T).
21+
Module Type QuotationOfMakeWithLeibniz (T : OrderedTypeWithLeibniz) (M : MSetList.MakeWithLeibnizSig T).
2522
Include QuotationOfMake T M.
2623
#[export] Declare Instance qeq_leibniz_list : quotation_of M.eq_leibniz_list.
2724
#[export] Declare Instance qeq_leibniz : quotation_of M.eq_leibniz.

0 commit comments

Comments
 (0)