Skip to content

Commit 2a29a06

Browse files
authored
Merge pull request #466 from math-comp/fix-warn
remove typechecking warnings
2 parents c58f776 + 9515dcd commit 2a29a06

File tree

4 files changed

+7
-7
lines changed

4 files changed

+7
-7
lines changed

tests/unit/close_hole_term.v

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -3,7 +3,7 @@ From elpi Require Import elpi.
33
From Coq Require Export Setoid.
44

55
Elpi Query HB.instance lp:{{
6-
X = app [{{list}}, Y],
6+
X = app [{{list}}, Y_],
77
% X needs to be typechecked here to get rid of the hole for the type of Y
88
coq.typecheck X _ ok,
99
abstract-holes.main X Z,

tests/unit/enrich_type.v

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -9,19 +9,19 @@ Elpi Query HB.structure lp:{{
99

1010
Elpi Query HB.structure lp:{{
1111
saturate-type-constructor {{list}} X,
12-
std.assert! (X = app [{{list}}, Y]) "wrong enriched type"
12+
std.assert! (X = app [{{list}}, Y_]) "wrong enriched type"
1313
}}.
1414

1515
Elpi Query HB.structure lp:{{
1616
Y = (x \ (y \ {{(prod (list lp:x) (list lp:y))}})),
1717
saturate-type-constructor (Y _ _) X,
18-
std.assert! (X = (app [{{prod}}, (app[{{list}},X1]), app[{{list}},C]])) "wrong enriched type"
18+
std.assert! (X = (app [{{prod}}, (app[{{list}},X1_]), app[{{list}},C_]])) "wrong enriched type"
1919
}}.
2020

2121
Class Inj {A B} (R : relation A) (S : relation B) (f : A -> B) : Prop :=
2222
inj x y : S (f x) (f y) -> R x y.
2323

2424
Elpi Query HB.structure lp:{{
2525
saturate-type-constructor {{Inj}} X,
26-
std.assert! (X = app [(global (const Inj)), A, B, R, S, F]) "wrong enriched type"
26+
std.assert! (X = app [(global (const Inj_)), A_, B_, R_, S_, F_]) "wrong enriched type"
2727
}}.

tests/unit/mixin_src_has_mixin_instance.v

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -13,7 +13,7 @@ HB.instance Definition nat_m2 : m2 nat := m2.Build nat 1.
1313

1414

1515
Elpi Query HB.instance lp:{{
16-
mixin-src->has-mixin-instance (mixin-src {{nat}} M1 {{nat_m1}}) Y,
16+
mixin-src->has-mixin-instance (mixin-src {{nat}} M1_ {{nat_m1}}) Y,
1717
Y = has-mixin-instance (cs-gref {{:gref nat}}) {{:gref m1.phant_axioms}} {{:gref nat_m1}}.
1818

1919
}}.
@@ -22,7 +22,7 @@ Section Test.
2222
Variable X:s1.type.
2323

2424
Elpi Query HB.instance lp:{{
25-
mixin-src->has-mixin-instance (mixin-src {{list X}} M1 {{i1 X}}) Y,
25+
mixin-src->has-mixin-instance (mixin-src {{list X}} M1_ {{i1 X}}) Y,
2626
Y = has-mixin-instance (cs-gref {{:gref list}}) {{:gref m1.phant_axioms}} {{:gref i1}}.
2727

2828
}}.

tests/unit/struct.v

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -8,7 +8,7 @@ HB.structure Definition foo1 := { A of is_foo (option nat) A & m1 A}.
88

99

1010
Elpi Query HB.structure lp:{{
11-
std.findall (has-mixin-instance _ _ _) H
11+
std.findall (has-mixin-instance _ _ _) H_
1212
}}.
1313

1414
(* here we don't have any declared instances but a clause is still created by the system :

0 commit comments

Comments
 (0)