Skip to content

Commit

Permalink
Fix minor stuffs in test-suite and translations
Browse files Browse the repository at this point in the history
  • Loading branch information
SimonBoulier committed Mar 3, 2020
1 parent f81e8a2 commit 00e2150
Show file tree
Hide file tree
Showing 5 changed files with 15 additions and 16 deletions.
20 changes: 13 additions & 7 deletions test-suite/_CoqProject
Original file line number Diff line number Diff line change
Expand Up @@ -9,6 +9,8 @@
-Q ../erasure/theories MetaCoq.Erasure
-R . MetaCoq.TestSuite

# list obtained with `ls -1 *.v`

bug1.v
bug2.v
bug5.v
Expand All @@ -20,19 +22,23 @@ case.v
castprop.v
# CheckerTest.v disabled
cofix.v
erasure_live_test.v
erasure_test.v
evars.v
extractable.v
hnf_ctor.v
issue27.v
issue28.v
letin.v
mutind.v
opaque.v
proj.v
run_in_tactic.v
safechecker_test.v
# test_term.v -> loaded in TypingTests.v
tmExistingInstance.v
tmInferInstance.v
TypingTests.v
unfold.v
univ.v
tmInferInstance.v
issue27.v
issue28.v
extractable.v
vs.v
erasure_test.v
safechecker_test.v
erasure_live_test.v
2 changes: 1 addition & 1 deletion test-suite/unfold.v
Original file line number Diff line number Diff line change
@@ -1,3 +1,3 @@
Require Import MetaCoq.Template.All.
Require Import MetaCoq.Template.All String.

Run TemplateProgram (tmBind (tmEval (unfold "negb") negb) tmPrint).
2 changes: 1 addition & 1 deletion translations/_CoqProject.in
Original file line number Diff line number Diff line change
Expand Up @@ -6,7 +6,7 @@ sigma.v
MiniHoTT.v
MiniHoTT_paths.v
translation_utils.v
#param_original.v
param_original.v
param_cheap_packed.v
param_generous_packed.v
#param_generous_unpacked.v
Expand Down
1 change: 0 additions & 1 deletion translations/param_original.v
Original file line number Diff line number Diff line change
Expand Up @@ -246,7 +246,6 @@ Module Id2.
Definition free_thm_myf : forall A x y p, myf A x y p = p
:= param_ID_identity myf myfᵗ.
End Id2.
*)



Expand Down
6 changes: 0 additions & 6 deletions translations/translation_utils.v
Original file line number Diff line number Diff line change
Expand Up @@ -184,12 +184,6 @@ Definition Implement {tsl : Translation} (ΣE : tsl_context)
end
end.

Definition body_constant_entry (e : constant_entry) : option term :=
match e with
| ParameterEntry _ => None
| DefinitionEntry {| definition_entry_body := t |} => Some t
end.


Definition ImplementExisting {tsl : Translation} (ΣE : tsl_context) (id : ident)
: TemplateMonad tsl_context :=
Expand Down

0 comments on commit 00e2150

Please sign in to comment.