Skip to content

Commit 644b830

Browse files
Import FInFun (#825)
* use RelationClasses instead of old Relations_1 (for rocq-prover/stdlib#152) * 'make test2' now builds in Rocq 9 with dev versions of Flocq and CompCert --------- Co-authored-by: Andres Erbsen <[email protected]>
1 parent 127aa73 commit 644b830

File tree

7 files changed

+11
-9
lines changed

7 files changed

+11
-9
lines changed

coq-ext-lib

fcf

msl/subtypes.v

Lines changed: 1 addition & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -3,12 +3,11 @@
33
*
44
*)
55

6+
Require Import Arith.
67
Require Import VST.msl.base.
78
Require Import VST.msl.ageable.
89
Require Import VST.msl.predicates_hered.
910

10-
Import Arith.
11-
1211
Local Open Scope pred.
1312

1413
Section Fash.

progs64/io_os_connection.v

Lines changed: 3 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -565,11 +565,13 @@ Section Invariants.
565565
intros Hin; apply in_combine_l in Hin; easy.
566566
Qed.
567567

568+
Require Import FinFun.
569+
568570
Lemma mkRecvEvents_NoDup : forall logIdx cs,
569571
NoDup (mkRecvEvents logIdx cs).
570572
Proof.
571573
unfold mkRecvEvents, enumerate; intros.
572-
apply FinFun.Injective_map_NoDup; auto using combine_NoDup, seq_NoDup.
574+
apply Injective_map_NoDup; auto using combine_NoDup, seq_NoDup.
573575
red; intros (? & ?) (? & ?); intros; inj; auto.
574576
Qed.
575577

zlist/list_solver.v

Lines changed: 3 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -1,3 +1,4 @@
1+
Require Import RelationClasses.
12
Require Import ZArith Znumtheory.
23
Require Import Coq.Lists.List.
34
Require Import Lia.
@@ -1030,8 +1031,8 @@ Section Sorted.
10301031
Variable A : Type.
10311032
Variable d : Inhabitant A.
10321033
Variable le : A -> A -> Prop.
1033-
Context {Hrefl : Relations_1.Reflexive A le}.
1034-
Context {Htrans : Relations_1.Transitive le}.
1034+
Context {Hrefl : Reflexive le}.
1035+
Context {Htrans : Transitive le}.
10351036

10361037
Definition sorted (l : list A) :=
10371038
forall i j, 0 <= i <= j /\ j < Zlength l -> le (Znth i l) (Znth j l).

0 commit comments

Comments
 (0)