File tree Expand file tree Collapse file tree 11 files changed +15
-36
lines changed
quotation/theories/ToTemplate Expand file tree Collapse file tree 11 files changed +15
-36
lines changed Original file line number Diff line number Diff line change 11From 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 .
33From MetaCoq.Quotation.ToTemplate Require Import Init.
44From MetaCoq.Quotation.ToTemplate Require Import (hints) Coq.Numbers Coq.Init Coq.Lists.
55From MetaCoq.Quotation.ToTemplate.QuotationOf.Coq.Structures Require Import OrdersAlt.Sig.
Original file line number Diff line number Diff line change 11From Coq Require Import MSetInterface MSetList MSetAVL MSetFacts MSetProperties MSetDecide.
2+ From MetaCoq.Utils Require Import MCMSets.
23From MetaCoq.Quotation.ToTemplate Require Import Init.
34From MetaCoq.Quotation.ToTemplate Require Import (hints) Coq.Numbers Coq.Init Coq.Lists.
45From MetaCoq.Quotation.ToTemplate.QuotationOf.Coq.Structures Require Import Orders.Sig.
Original file line number Diff line number Diff line change 11From Coq.FSets Require Import FMapAVL.
22From Coq.Structures Require Import Equalities OrdersAlt.
3+ From MetaCoq.Utils Require Import MCFSets.
34From MetaCoq.Quotation.ToTemplate Require Import Init.
45From MetaCoq.Quotation.ToTemplate.QuotationOf.Coq.Structures Require Import OrdersAlt.Sig.
56From MetaCoq.Quotation.ToTemplate.QuotationOf.Coq.FSets Require Import FMapList.Sig.
67Import List.ListNotations.
78Local Open Scope list_scope.
89
910Module 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.
Original file line number Diff line number Diff line change 11From Coq.FSets Require Import FMapFacts.
22From Coq.Structures Require Import Orders.
3+ From MetaCoq.Utils Require Import MCFSets.
34From MetaCoq.Quotation.ToTemplate Require Import Init.
45
56Module 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.
Original file line number Diff line number Diff line change 11From Coq.FSets Require Import FMapList.
22From Coq.Structures Require Import Equalities OrdersAlt.
3+ From MetaCoq.Utils Require Import MCFSets.
34From MetaCoq.Quotation.ToTemplate Require Import Init.
45From MetaCoq.Quotation.ToTemplate.QuotationOf.Coq.Structures Require Import OrdersAlt.Sig.
56Import List.ListNotations.
67Local Open Scope list_scope.
78
89Module 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.
Original file line number Diff line number Diff line change 11From Coq.Structures Require Import Orders.
22From Coq.MSets Require Import MSetAVL.
3+ From MetaCoq.Utils Require Import MCMSets.
34From MetaCoq.Quotation.ToTemplate Require Import Init.
45
56Module 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.
1110End MSetAVL.
Original file line number Diff line number Diff line change 11From Coq.MSets Require Import MSetInterface MSetDecide.
2+ From MetaCoq.Utils Require Import MCMSets.
23From MetaCoq.Quotation.ToTemplate Require Import Init.
34
45Module 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.
Original file line number Diff line number Diff line change 11From Coq.MSets Require Import MSetFacts.
2+ From MetaCoq.Utils Require Import MCMSets.
23From MetaCoq.Quotation.ToTemplate Require Import Init.
34
45Module 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.
Original file line number Diff line number Diff 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.
2222End QuotationOfSetsOn.
2323Module 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.
Original file line number Diff line number Diff line change 11From Coq.Structures Require Import Equalities Orders.
22From Coq.MSets Require Import MSetList.
3+ From MetaCoq.Utils Require Import MCMSets.
34From MetaCoq.Quotation.ToTemplate Require Import Init.
45From MetaCoq.Quotation.ToTemplate.QuotationOf.Coq.MSets Require Import MSetInterface.Sig.
56
@@ -13,15 +14,11 @@ Module Type QuotationOfSWithLeibniz (S : SWithLeibniz).
1314End QuotationOfSWithLeibniz.
1415
1516Module 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.
You can’t perform that action at this time.
0 commit comments