Skip to content

Commit

Permalink
fix tests
Browse files Browse the repository at this point in the history
  • Loading branch information
gares committed Nov 14, 2024
1 parent 73056be commit cf6b942
Show file tree
Hide file tree
Showing 7 changed files with 7 additions and 13 deletions.
1 change: 0 additions & 1 deletion apps/coercion/README.md
Original file line number Diff line number Diff line change
Expand Up @@ -36,7 +36,6 @@ coercion _ {{ True }} {{ Prop }} {{ bool }} {{ true }}.
coercion _ {{ False }} {{ Prop }} {{ bool }} {{ false }}.
}}.
Elpi Typecheck coercion. (* checks the elpi program is OK *)
Check True && False.
```
Expand Down
2 changes: 0 additions & 2 deletions apps/coercion/tests/coercion.t/test.v
Original file line number Diff line number Diff line change
Expand Up @@ -8,7 +8,6 @@ coercion _ {{ True }} {{ Prop }} {{ bool }} {{ true }}.
coercion _ {{ False }} {{ Prop }} {{ bool }} {{ false }}.

}}.
Elpi Typecheck coercion.

Check True && False.

Expand All @@ -22,7 +21,6 @@ coercion _ N {{ nat }} {{ ringType_sort lp:R }} {{ natmul lp:R lp:N }} :-
coq.typecheck R {{ ringType }} ok.

}}.
Elpi Typecheck coercion.

Section TestNatMul.

Expand Down
3 changes: 1 addition & 2 deletions apps/coercion/tests/coercion_open.t/test.v
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,7 @@ From Coq Require Import Arith ssreflect.

Ltac my_solver := trivial with arith.

Elpi Accumulate coercion.db lp:{{
Elpi Accumulate coercion lp:{{

coercion _ X Ty {{ @sig lp:Ty lp:P }} Solution :- std.do! [
% we unfold letins since the solve is dumb
Expand All @@ -17,7 +17,6 @@ coercion _ X Ty {{ @sig lp:Ty lp:P }} Solution :- std.do! [
].

}}.
Elpi Typecheck coercion.

Goal {x : nat | x > 0}.
apply: 3.
Expand Down
1 change: 0 additions & 1 deletion apps/cs/README.md
Original file line number Diff line number Diff line change
Expand Up @@ -38,7 +38,6 @@ cs _ {{ sort lp:Sol }} {{ nat }} :-
Sol = {{ Build_S nat }}.
}}.
Elpi Typecheck canonical_solution.
Check eq_refl _ : (sort _) = nat.
```
1 change: 0 additions & 1 deletion apps/cs/tests/cs.t.disabled_broken_8.19/test.v
Original file line number Diff line number Diff line change
Expand Up @@ -9,7 +9,6 @@ Elpi Accumulate canonical_solution lp:{{
cs _ {{ sort lp:T }} {{ @id lp:T }} {{ Build_S lp:T (@id lp:T) }}.

}}.
Elpi Typecheck canonical_solution.

Check 1.
Check eq_refl _ : (sort nat _) = @id nat.
Expand Down
1 change: 0 additions & 1 deletion apps/derive/README.md
Original file line number Diff line number Diff line change
Expand Up @@ -575,7 +575,6 @@ From elpi.apps Require Export
...
myder (* new derivation *)
.
Elpi Typecheck derive.
```

So when the user `Import`s `better_std` he gets a fully loaded `derive`.
Expand Down
11 changes: 6 additions & 5 deletions examples/tutorial_coq_elpi_tactic.v
Original file line number Diff line number Diff line change
Expand Up @@ -92,11 +92,12 @@ is stored in the .vo file (the external file does not need to be installed).
We invite the reader to look up the description of data bases in the tutorial
about commands.
Once all the code is accumulated `Elpi Typecheck` verifies that the
code does not contain the most frequent kind of mistakes. This command
considers some mistakes minor and only warns about them. You can
pass `-w +elpi.typecheck` to `coqc` to turn these warnings into errors.
When some code is accumulated Elpi verifies that the
code does not contain the most frequent kind of mistakes, via some
type checking and linting. Some mistakes are minor and Elpi only warns about
them. You can pass `-w +elpi.typecheck` to `coqc` to turn these warnings into
errors.
The entry point for tactics is called :builtin:`solve` which maps a :type:`goal`
into a list of :type:`sealed-goal` (representing subgoals).
Expand Down

0 comments on commit cf6b942

Please sign in to comment.