File tree Expand file tree Collapse file tree 7 files changed +7
-13
lines changed
tests/cs.t.disabled_broken_8.19 Expand file tree Collapse file tree 7 files changed +7
-13
lines changed Original file line number Diff line number Diff line change @@ -36,7 +36,6 @@ coercion _ {{ True }} {{ Prop }} {{ bool }} {{ true }}.
36
36
coercion _ {{ False }} {{ Prop }} {{ bool }} {{ false }}.
37
37
38
38
}}.
39
- Elpi Typecheck coercion. (* checks the elpi program is OK *)
40
39
41
40
Check True && False.
42
41
```
Original file line number Diff line number Diff line change @@ -8,7 +8,6 @@ coercion _ {{ True }} {{ Prop }} {{ bool }} {{ true }}.
8
8
coercion _ {{ False }} {{ Prop }} {{ bool }} {{ false }}.
9
9
10
10
}}.
11
- Elpi Typecheck coercion.
12
11
13
12
Check True && False.
14
13
@@ -22,7 +21,6 @@ coercion _ N {{ nat }} {{ ringType_sort lp:R }} {{ natmul lp:R lp:N }} :-
22
21
coq.typecheck R {{ ringType }} ok.
23
22
24
23
}}.
25
- Elpi Typecheck coercion.
26
24
27
25
Section TestNatMul.
28
26
Original file line number Diff line number Diff line change @@ -4,7 +4,7 @@ From Coq Require Import Arith ssreflect.
4
4
5
5
Ltac my_solver := trivial with arith.
6
6
7
- Elpi Accumulate coercion.db lp:{{
7
+ Elpi Accumulate coercion lp:{{
8
8
9
9
coercion _ X Ty {{ @sig lp:Ty lp:P }} Solution :- std.do! [
10
10
% we unfold letins since the solve is dumb
@@ -17,7 +17,6 @@ coercion _ X Ty {{ @sig lp:Ty lp:P }} Solution :- std.do! [
17
17
].
18
18
19
19
}}.
20
- Elpi Typecheck coercion.
21
20
22
21
Goal {x : nat | x > 0}.
23
22
apply: 3.
Original file line number Diff line number Diff line change @@ -38,7 +38,6 @@ cs _ {{ sort lp:Sol }} {{ nat }} :-
38
38
Sol = {{ Build_S nat }}.
39
39
40
40
}}.
41
- Elpi Typecheck canonical_solution.
42
41
43
42
Check eq_refl _ : (sort _) = nat.
44
43
```
Original file line number Diff line number Diff line change @@ -9,7 +9,6 @@ Elpi Accumulate canonical_solution lp:{{
9
9
cs _ {{ sort lp:T }} {{ @id lp:T }} {{ Build_S lp:T (@id lp:T) }}.
10
10
11
11
}}.
12
- Elpi Typecheck canonical_solution.
13
12
14
13
Check 1.
15
14
Check eq_refl _ : (sort nat _) = @id nat.
Original file line number Diff line number Diff line change @@ -575,7 +575,6 @@ From elpi.apps Require Export
575
575
...
576
576
myder (* new derivation *)
577
577
.
578
- Elpi Typecheck derive.
579
578
```
580
579
581
580
So when the user ` Import ` s ` better_std ` he gets a fully loaded ` derive ` .
Original file line number Diff line number Diff line change @@ -92,11 +92,12 @@ is stored in the .vo file (the external file does not need to be installed).
92
92
We invite the reader to look up the description of data bases in the tutorial
93
93
about commands.
94
94
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
+
100
101
The entry point for tactics is called :builtin:`solve` which maps a :type:`goal`
101
102
into a list of :type:`sealed-goal` (representing subgoals).
102
103
You can’t perform that action at this time.
0 commit comments