Skip to content

Commit de9bba2

Browse files
committed
Remove unused Stdlib dependencies in tests
1 parent 225636a commit de9bba2

40 files changed

+172
-50
lines changed

apps/coercion/tests/test.v

Lines changed: 1 addition & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -1,6 +1,5 @@
11
From elpi.apps Require Import coercion.
22
#[warning="-deprecated-from-Coq"]
3-
From Coq Require Import Bool.
43

54
Elpi Accumulate coercion.db lp:{{
65

@@ -9,7 +8,7 @@ coercion _ {{ False }} {{ Prop }} {{ bool }} {{ false }}.
98

109
}}.
1110

12-
Check True && False.
11+
Check andb True False.
1312

1413
Parameter ringType : Type.
1514
Parameter ringType_sort : ringType -> Type.

apps/coercion/tests/test_open.v

Lines changed: 2 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -1,8 +1,7 @@
11
From elpi.apps Require Import coercion.
2-
#[warning="-deprecated-from-Coq"]
3-
From Coq Require Import Arith ssreflect.
2+
From elpi.core Require Import ssreflect.
43

5-
Ltac my_solver := trivial with arith.
4+
Ltac my_solver := try ((repeat apply: le_n_S); apply: le_0_n).
65

76
Elpi Accumulate coercion lp:{{
87

apps/derive/examples/usage.v

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -2,7 +2,6 @@
22
This example shows how to use derive
33
*)
44

5-
From Coq Require Import Bool.
65
From elpi.apps Require Import derive.std.
76
Set Uniform Inductive Parameters.
87

apps/derive/tests/test_bcongr.v

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -1,3 +1,4 @@
1+
From elpi.core Require Import Bool.
12
From elpi.apps Require Import derive.bcongr.
23

34
From elpi.apps Require Import test_derive_corelib test_projK.

apps/derive/tests/test_derive_corelib.v

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -1,6 +1,6 @@
11
(* Some standard data types using different features *)
2-
From Coq Require Uint63.
3-
From Coq Require Floats.
2+
From elpi.core Require PrimInt63.
3+
From elpi.core Require PrimFloat.
44

55
Module Coverage.
66

@@ -68,7 +68,7 @@ Inductive large :=
6868
| K25(_ : unit) (_ : unit) (_ : unit) (_ : unit) (_ : unit) (_ : unit) (_ : unit) (_ : unit) (_ : unit) (_ : unit) (_ : unit) (_ : unit) (_ : unit) (_ : unit) (_ : unit) (_ : unit) (_ : unit) (_ : unit) (_ : unit) (_ : unit) (_ : unit) (_ : unit) (_ : unit) (_ : unit) (_ : unit)
6969
| K26(_ : unit) (_ : unit) (_ : unit) (_ : unit) (_ : unit) (_ : unit) (_ : unit) (_ : unit) (_ : unit) (_ : unit) (_ : unit) (_ : unit) (_ : unit) (_ : unit) (_ : unit) (_ : unit) (_ : unit) (_ : unit) (_ : unit) (_ : unit) (_ : unit) (_ : unit) (_ : unit) (_ : unit) (_ : unit) (_ : unit).
7070

71-
Inductive prim_int := PI (i : Uint63.int).
71+
Inductive prim_int := PI (i : PrimInt63.int).
7272
Inductive prim_float := PF (f : PrimFloat.float).
7373

7474
Record fo_record := { f1 : peano; f2 : unit; }.

apps/derive/tests/test_eqb.v

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -41,7 +41,7 @@ Elpi derive.eqb alias.
4141

4242
End Coverage.
4343
Import Coverage.
44-
Import PArith.
44+
From elpi.core Require Import PosDef.
4545

4646
Notation eq_test T := (T -> T -> bool).
4747
Notation eq_test2 T1 T2 := (T1 -> T2 -> bool).

apps/derive/tests/test_eqbOK.v

Lines changed: 5 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -1,3 +1,4 @@
1+
From elpi.core Require Import Bool.
12
From elpi.apps Require Import derive.eqbOK.
23

34
From elpi.apps.derive.tests Require Import test_derive_corelib test_eqb test_eqbcorrect.
@@ -48,7 +49,7 @@ End Coverage.
4849

4950
Import Coverage.
5051

51-
Redirect "tmp" Check peano_eqb_OK : forall n m, Bool.reflect (n = m) (peano_eqb n m).
52-
Redirect "tmp" Check seq_eqb_OK : forall A eqA (h : forall a1 a2 : A, Bool.reflect (a1 = a2) (eqA a1 a2)) l1 l2, Bool.reflect (l1 = l2) (seq_eqb A eqA l1 l2).
53-
Redirect "tmp" Check ord_eqb_OK : forall n (o1 o2 : ord n), Bool.reflect (o1 = o2) (ord_eqb n n o1 o2).
54-
Redirect "tmp" Check alias_eqb_OK : forall x y : alias, Bool.reflect (x = y) (alias_eqb x y).
52+
Redirect "tmp" Check peano_eqb_OK : forall n m, Datatypes.reflect (n = m) (peano_eqb n m).
53+
Redirect "tmp" Check seq_eqb_OK : forall A eqA (h : forall a1 a2 : A, Datatypes.reflect (a1 = a2) (eqA a1 a2)) l1 l2, Datatypes.reflect (l1 = l2) (seq_eqb A eqA l1 l2).
54+
Redirect "tmp" Check ord_eqb_OK : forall n (o1 o2 : ord n), Datatypes.reflect (o1 = o2) (ord_eqb n n o1 o2).
55+
Redirect "tmp" Check alias_eqb_OK : forall x y : alias, Datatypes.reflect (x = y) (alias_eqb x y).

apps/derive/tests/test_fields.v

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -38,7 +38,7 @@ Elpi derive.fields val.
3838
End Coverage.
3939

4040
Import Coverage.
41-
Import PArith.
41+
From elpi.core Require Import PosDef.
4242

4343
Redirect "tmp" Check empty_fields_t : positive -> Type.
4444
Redirect "tmp" Check empty_fields : forall (n:empty), empty_fields_t (empty_tag n).

apps/derive/tests/test_tag.v

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -39,7 +39,7 @@ Elpi derive.tag val.
3939
End Coverage.
4040

4141
Import Coverage.
42-
Import PArith.
42+
From elpi.core Require Import PosDef.
4343

4444
Local Notation tag X := (X -> positive).
4545

apps/eltac/tests/test_apply.v

Lines changed: 4 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -5,7 +5,9 @@ Proof.
55
eltac.apply H.
66
Qed.
77

8+
Axiom add_comm : forall x y, x + y = y + x.
9+
810
Goal (3 + 4 = 4 + 3).
911
Proof.
10-
eltac.apply PeanoNat.Nat.add_comm.
11-
Qed.
12+
eltac.apply add_comm.
13+
Qed.

0 commit comments

Comments
 (0)