Skip to content

Commit 5827121

Browse files
authored
Merge pull request #662 from proux01/coq_19310
Adapt to rocq-prover/rocq#19310
2 parents 9c9823d + 6124e37 commit 5827121

File tree

4 files changed

+7
-4
lines changed

4 files changed

+7
-4
lines changed

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

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

45
Elpi Accumulate coercion.db lp:{{

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

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -1,4 +1,5 @@
11
From elpi.apps Require Import coercion.
2+
#[warning="-deprecated-from-Coq"]
23
From Coq Require Import Arith ssreflect.
34

45
Ltac my_solver := trivial with arith.

apps/tc/elpi/tc_aux.elpi

Lines changed: 2 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -93,7 +93,8 @@ namespace tc {
9393
if (tc.is-option-active tc.oTC-clauseNameShortName)
9494
(Path = "")
9595
(coq.gref->path Gr [Hd | Tl],
96-
std.fold Tl Hd (x\acc\r\ r is acc ^ "." ^ x) Path',
96+
if (Hd = "Coq") (Hd' = "Stdlib") (Hd' = Hd),
97+
std.string.concat "." [Hd'|Tl] Path',
9798
Path is Path' ^ ".tc-"),
9899
% CAVEAT : Non-ascii caractars can't be part of a pred
99100
% name, we replace ö with o

apps/tc/tests/bigTest.v

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -882,7 +882,7 @@ instances *)
882882
Section prod_setoid.
883883
Context `{Equiv A, Equiv B}.
884884
Elpi Accumulate TC.Solver lp:{{
885-
shorten tc-Coq.Classes.RelationClasses.{tc-Equivalence}.
885+
shorten tc-Stdlib.Classes.RelationClasses.{tc-Equivalence}.
886886
:after "lastHook"
887887
tc-Equivalence A RA R :-
888888
RA = {{@equiv _ (@prod_equiv _ _ _ _)}},
@@ -910,7 +910,7 @@ Section prod_setoid.
910910
std.map L1 remove_equiv_prod_equiv L2.
911911
remove_equiv_prod_equiv A A.
912912

913-
shorten tc-Coq.Classes.Morphisms.{tc-Proper}.
913+
shorten tc-Stdlib.Classes.Morphisms.{tc-Proper}.
914914

915915
:after "lastHook"
916916
tc-Proper A B C R :-
@@ -1043,7 +1043,7 @@ Elpi Accumulate TC.Solver lp:{{
10431043
std.map L1 remove_equiv_sum_equiv L2.
10441044
remove_equiv_sum_equiv A A.
10451045

1046-
shorten tc-Coq.Classes.Morphisms.{tc-Proper}.
1046+
shorten tc-Stdlib.Classes.Morphisms.{tc-Proper}.
10471047
:after "lastHook"
10481048
tc-Proper A B C R :-
10491049
B = {{ @respectful _ _ _ _ }},

0 commit comments

Comments
 (0)