Skip to content

Commit

Permalink
Merge pull request #148 from proux01/stdlib_repo
Browse files Browse the repository at this point in the history
Adapt to coq/coq#19530
  • Loading branch information
jwiegley authored Sep 17, 2024
2 parents 268c570 + 04da82e commit b1033ae
Show file tree
Hide file tree
Showing 7 changed files with 15 additions and 17 deletions.
4 changes: 2 additions & 2 deletions Instance/Lambda/Ltac.v
Original file line number Diff line number Diff line change
@@ -1,5 +1,5 @@
Require Import Coq.Unicode.Utf8.
Require Import Coq.Program.Program.
From Coq Require Import Utf8.

Check warning on line 1 in Instance/Lambda/Ltac.v

View workflow job for this annotation

GitHub Actions / build (coqorg/coq:dev)

"From Coq" has been replaced by "From Stdlib".
From Coq Require Import Program.

Check warning on line 2 in Instance/Lambda/Ltac.v

View workflow job for this annotation

GitHub Actions / build (coqorg/coq:dev)

"From Coq" has been replaced by "From Stdlib".

Local Set Warnings "-deprecated-notation".

Expand Down
4 changes: 2 additions & 2 deletions Lib/Foundation.v
Original file line number Diff line number Diff line change
@@ -1,5 +1,5 @@
Require Export Coq.Program.Program.
Require Export Coq.Classes.CMorphisms.
From Coq Require Export Program.

Check warning on line 1 in Lib/Foundation.v

View workflow job for this annotation

GitHub Actions / build (coqorg/coq:dev)

"From Coq" has been replaced by "From Stdlib".
From Coq Require Export CMorphisms.

Check warning on line 2 in Lib/Foundation.v

View workflow job for this annotation

GitHub Actions / build (coqorg/coq:dev)

"From Coq" has been replaced by "From Stdlib".

Generalizable All Variables.
Set Primitive Projections.
Expand Down
6 changes: 3 additions & 3 deletions Lib/MapDecide.v
Original file line number Diff line number Diff line change
@@ -1,6 +1,6 @@
Require Import Coq.NArith.NArith.
Require Import Coq.FSets.FMaps.
Require Import Coq.micromega.Lia.
From Coq Require Import NArith.
From Coq Require Import FMaps.
From Coq Require Import Lia.

(* Override ++> notation with the crelation-based version. *)
#[local] Set Warnings "-notation-overridden".
Expand Down
4 changes: 1 addition & 3 deletions Theory/Coq/List.v
Original file line number Diff line number Diff line change
Expand Up @@ -399,9 +399,7 @@ Instance List_Applicative : Applicative list := {
ap := @list_ap
}.

Require Import
Coq.Relations.Relations
Coq.Reals.ROrderedType.
From Coq Require Import Relations ROrderedType.

Require Export Coq.Lists.List.

Expand Down
4 changes: 2 additions & 2 deletions Theory/Coq/Map.v
Original file line number Diff line number Diff line change
@@ -1,5 +1,5 @@
Require Import Coq.Lists.List.
Require Import Coq.micromega.Lia.
From Coq Require Import List.
From Coq Require Import Lia.

From Equations Require Import Equations.
Set Equations With UIP.
Expand Down
6 changes: 3 additions & 3 deletions Theory/Metacategory.v
Original file line number Diff line number Diff line change
@@ -1,7 +1,7 @@
Require Import Coq.Structures.DecidableTypeEx.
Require Import Coq.FSets.FMapFacts.
From Coq Require Import DecidableTypeEx.
From Coq Require Import FMapFacts.
Require Import Category.Lib.FMapExt.
Require Import Coq.Arith.PeanoNat.
From Coq Require Import PeanoNat.

(* Override ++> notation with the crelation-based version. *)
#[local] Set Warnings "-notation-overridden".
Expand Down
4 changes: 2 additions & 2 deletions Theory/Metacategory/ArrowsOnly.v
Original file line number Diff line number Diff line change
@@ -1,5 +1,5 @@
Require Import Coq.NArith.NArith.
Require Import Coq.micromega.Lia.
From Coq Require Import NArith.
From Coq Require Import Lia.

Require Import Category.Lib.
Require Import Category.Lib.MapDecide.
Expand Down

0 comments on commit b1033ae

Please sign in to comment.