Skip to content

Commit

Permalink
Clean up some import lists
Browse files Browse the repository at this point in the history
  • Loading branch information
pi8027 committed Nov 13, 2024
1 parent 1fc1c88 commit 5e1d123
Show file tree
Hide file tree
Showing 3 changed files with 6 additions and 6 deletions.
6 changes: 3 additions & 3 deletions theories/heaps.v
Original file line number Diff line number Diff line change
Expand Up @@ -15,11 +15,11 @@
along with this program. If not, see <http://www.gnu.org/licenses/>.
*)

From Coq Require Import Eqdep.

Check warning on line 18 in theories/heaps.v

View workflow job for this annotation

GitHub Actions / build (mathcomp/mathcomp-dev:coq-dev)

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

Check warning on line 18 in theories/heaps.v

View workflow job for this annotation

GitHub Actions / build (mathcomp/mathcomp:2.2.0-coq-dev)

"From Coq" has been replaced by "From Stdlib".
From HB Require Import structures.
From mathcomp Require Import ssreflect ssrfun ssrnat div ssrbool seq.
From mathcomp Require Import ssreflect ssrfun ssrbool eqtype ssrnat seq div.
From LemmaOverloading Require Import prelude finmap ordtype.
From mathcomp Require Import path eqtype.
Require Import Eqdep.
From mathcomp Require Import path.
Set Implicit Arguments.
Unset Strict Implicit.
Unset Printing Implicit Defensive.
Expand Down
4 changes: 2 additions & 2 deletions theories/prelude.v
Original file line number Diff line number Diff line change
Expand Up @@ -15,8 +15,8 @@
along with this program. If not, see <http://www.gnu.org/licenses/>.
*)

Require Import Eqdep ClassicalFacts.
From mathcomp Require Import ssreflect ssrbool eqtype ssrfun seq.
From Coq Require Import Eqdep ClassicalFacts.

Check warning on line 18 in theories/prelude.v

View workflow job for this annotation

GitHub Actions / build (mathcomp/mathcomp-dev:coq-dev)

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

Check warning on line 18 in theories/prelude.v

View workflow job for this annotation

GitHub Actions / build (mathcomp/mathcomp:2.2.0-coq-dev)

"From Coq" has been replaced by "From Stdlib".
From mathcomp Require Import ssreflect ssrfun ssrbool eqtype seq.
Set Implicit Arguments.
Unset Strict Implicit.
Unset Printing Implicit Defensive.
Expand Down
2 changes: 1 addition & 1 deletion theories/rels.v
Original file line number Diff line number Diff line change
Expand Up @@ -15,8 +15,8 @@
along with this program. If not, see <http://www.gnu.org/licenses/>.
*)

From Coq Require Import Setoid.

Check warning on line 18 in theories/rels.v

View workflow job for this annotation

GitHub Actions / build (mathcomp/mathcomp-dev:coq-dev)

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

Check warning on line 18 in theories/rels.v

View workflow job for this annotation

GitHub Actions / build (mathcomp/mathcomp:2.2.0-coq-dev)

"From Coq" has been replaced by "From Stdlib".
From mathcomp Require Import ssreflect ssrfun ssrbool seq.
Require Import Setoid.
Set Implicit Arguments.
Unset Strict Implicit.
Unset Printing Implicit Defensive.
Expand Down

0 comments on commit 5e1d123

Please sign in to comment.