Skip to content

Commit 9ebf370

Browse files
committed
Refactor import for Coq_Dep
1 parent 87fe610 commit 9ebf370

File tree

3 files changed

+7
-2
lines changed

3 files changed

+7
-2
lines changed

apps/tc/theories/add_commands.v

Lines changed: 2 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -3,6 +3,7 @@
33

44
From elpi.apps Require Import db.
55

6+
From elpi.apps.tc Extra Dependency "tc_aux.elpi" as tc_aux.
67
From elpi.apps.tc Extra Dependency "compiler.elpi" as compiler.
78
From elpi.apps.tc Extra Dependency "parser_addInstances.elpi" as parser_addInstances.
89
From elpi.apps.tc Extra Dependency "solver.elpi" as solver.
@@ -57,8 +58,8 @@ Elpi Typecheck.
5758
Elpi Command TC.AddHook.
5859
Elpi Accumulate Db tc.db.
5960
Elpi Accumulate Db tc_options.db.
61+
Elpi Accumulate File tc_aux.
6062
Elpi Accumulate lp:{{
61-
accumulate elpi/tc_aux.
6263
pred addHook i:grafting, i:string.
6364
addHook Grafting NewName :-
6465
@global! => add-tc-db NewName Grafting (hook NewName).

apps/tc/theories/db.v

Lines changed: 3 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -3,6 +3,9 @@
33

44
From elpi Require Import elpi.
55

6+
From elpi.apps.tc Extra Dependency "base.elpi".
7+
From elpi.apps.tc Extra Dependency "tc_aux.elpi".
8+
69
(*
710
tc_option.db contains the set of options used by the solver of tc.
811
all the options are set to false by default

apps/tc/theories/tc.v

Lines changed: 2 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -3,6 +3,7 @@
33

44
Declare ML Module "coq-elpi-tc.plugin".
55

6+
From elpi.apps.tc Extra Dependency "tc_aux.elpi" as tc_aux.
67
From elpi.apps.tc Extra Dependency "compiler.elpi" as compiler.
78
From elpi.apps.tc Extra Dependency "solver.elpi" as solver.
89
From elpi.apps.tc Extra Dependency "create_tc_predicate.elpi" as create_tc_predicate.
@@ -81,8 +82,8 @@ Elpi Typecheck.
8182
Elpi Command TC.Set_deterministic.
8283
Elpi Accumulate Db tc.db.
8384
Elpi Accumulate Db tc_options.db.
85+
Elpi Accumulate File tc_aux.
8486
Elpi Accumulate lp:{{
85-
accumulate elpi/tc_aux.
8687
main [str ClassStr] :-
8788
coq.locate ClassStr ClassGR,
8889
std.assert! (coq.TC.class? ClassGR) "Should pass the name of a type class",

0 commit comments

Comments
 (0)