Skip to content

Commit cf6b942

Browse files
committed
fix tests
1 parent 73056be commit cf6b942

File tree

7 files changed

+7
-13
lines changed

7 files changed

+7
-13
lines changed

apps/coercion/README.md

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -36,7 +36,6 @@ coercion _ {{ True }} {{ Prop }} {{ bool }} {{ true }}.
3636
coercion _ {{ False }} {{ Prop }} {{ bool }} {{ false }}.
3737
3838
}}.
39-
Elpi Typecheck coercion. (* checks the elpi program is OK *)
4039
4140
Check True && False.
4241
```

apps/coercion/tests/coercion.t/test.v

Lines changed: 0 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -8,7 +8,6 @@ coercion _ {{ True }} {{ Prop }} {{ bool }} {{ true }}.
88
coercion _ {{ False }} {{ Prop }} {{ bool }} {{ false }}.
99

1010
}}.
11-
Elpi Typecheck coercion.
1211

1312
Check True && False.
1413

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

2423
}}.
25-
Elpi Typecheck coercion.
2624

2725
Section TestNatMul.
2826

apps/coercion/tests/coercion_open.t/test.v

Lines changed: 1 addition & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -4,7 +4,7 @@ From Coq Require Import Arith ssreflect.
44

55
Ltac my_solver := trivial with arith.
66

7-
Elpi Accumulate coercion.db lp:{{
7+
Elpi Accumulate coercion lp:{{
88

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

1919
}}.
20-
Elpi Typecheck coercion.
2120

2221
Goal {x : nat | x > 0}.
2322
apply: 3.

apps/cs/README.md

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -38,7 +38,6 @@ cs _ {{ sort lp:Sol }} {{ nat }} :-
3838
Sol = {{ Build_S nat }}.
3939
4040
}}.
41-
Elpi Typecheck canonical_solution.
4241
4342
Check eq_refl _ : (sort _) = nat.
4443
```

apps/cs/tests/cs.t.disabled_broken_8.19/test.v

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -9,7 +9,6 @@ Elpi Accumulate canonical_solution lp:{{
99
cs _ {{ sort lp:T }} {{ @id lp:T }} {{ Build_S lp:T (@id lp:T) }}.
1010

1111
}}.
12-
Elpi Typecheck canonical_solution.
1312

1413
Check 1.
1514
Check eq_refl _ : (sort nat _) = @id nat.

apps/derive/README.md

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -575,7 +575,6 @@ From elpi.apps Require Export
575575
...
576576
myder (* new derivation *)
577577
.
578-
Elpi Typecheck derive.
579578
```
580579

581580
So when the user `Import`s `better_std` he gets a fully loaded `derive`.

examples/tutorial_coq_elpi_tactic.v

Lines changed: 6 additions & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -92,11 +92,12 @@ is stored in the .vo file (the external file does not need to be installed).
9292
We invite the reader to look up the description of data bases in the tutorial
9393
about commands.
9494
95-
Once all the code is accumulated `Elpi Typecheck` verifies that the
96-
code does not contain the most frequent kind of mistakes. This command
97-
considers some mistakes minor and only warns about them. You can
98-
pass `-w +elpi.typecheck` to `coqc` to turn these warnings into errors.
99-
95+
When some code is accumulated Elpi verifies that the
96+
code does not contain the most frequent kind of mistakes, via some
97+
type checking and linting. Some mistakes are minor and Elpi only warns about
98+
them. You can pass `-w +elpi.typecheck` to `coqc` to turn these warnings into
99+
errors.
100+
100101
The entry point for tactics is called :builtin:`solve` which maps a :type:`goal`
101102
into a list of :type:`sealed-goal` (representing subgoals).
102103

0 commit comments

Comments
 (0)