File tree Expand file tree Collapse file tree 3 files changed +7
-2
lines changed Expand file tree Collapse file tree 3 files changed +7
-2
lines changed Original file line number Diff line number Diff line change 33
44From elpi.apps Require Import db.
55
6+ From elpi.apps.tc Extra Dependency "tc_aux.elpi" as tc_aux.
67From elpi.apps.tc Extra Dependency "compiler.elpi" as compiler.
78From elpi.apps.tc Extra Dependency "parser_addInstances.elpi" as parser_addInstances.
89From elpi.apps.tc Extra Dependency "solver.elpi" as solver.
@@ -57,8 +58,8 @@ Elpi Typecheck.
5758Elpi Command TC.AddHook.
5859Elpi Accumulate Db tc.db.
5960Elpi Accumulate Db tc_options.db.
61+ Elpi Accumulate File tc_aux.
6062Elpi 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).
Original file line number Diff line number Diff line change 33
44From 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
Original file line number Diff line number Diff line change 33
44Declare ML Module "coq-elpi-tc.plugin".
55
6+ From elpi.apps.tc Extra Dependency "tc_aux.elpi" as tc_aux.
67From elpi.apps.tc Extra Dependency "compiler.elpi" as compiler.
78From elpi.apps.tc Extra Dependency "solver.elpi" as solver.
89From elpi.apps.tc Extra Dependency "create_tc_predicate.elpi" as create_tc_predicate.
@@ -81,8 +82,8 @@ Elpi Typecheck.
8182Elpi Command TC.Set_deterministic.
8283Elpi Accumulate Db tc.db.
8384Elpi Accumulate Db tc_options.db.
85+ Elpi Accumulate File tc_aux.
8486Elpi 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",
You can’t perform that action at this time.
0 commit comments