Skip to content

Commit

Permalink
Minimize imports
Browse files Browse the repository at this point in the history
  • Loading branch information
proux01 committed May 19, 2024
1 parent 3a2608b commit cbad9fb
Show file tree
Hide file tree
Showing 131 changed files with 139 additions and 199 deletions.
2 changes: 1 addition & 1 deletion proofs/arch/arch_decl.v
Original file line number Diff line number Diff line change
@@ -1,6 +1,6 @@
(* -------------------------------------------------------------------- *)
From HB Require Import structures.
From mathcomp Require Import all_ssreflect ssralg ssrnum.
From mathcomp Require Import ssreflect ssrfun ssrbool ssrnat eqtype ssralg.
From mathcomp Require Import word_ssrZ.
From Coq Require Import
Relation_Operators
Expand Down
2 changes: 1 addition & 1 deletion proofs/arch/arch_extra.v
Original file line number Diff line number Diff line change
@@ -1,6 +1,6 @@
(* -------------------------------------------------------------------- *)
From HB Require Import structures.
From mathcomp Require Import all_ssreflect ssralg ssrnum.
From mathcomp Require Import ssreflect ssrfun ssrbool eqtype.
Require Import xseq strings utils var type values sopn expr fexpr arch_decl.
Require Import compiler_util.

Expand Down
4 changes: 2 additions & 2 deletions proofs/arch/arch_sem.v
Original file line number Diff line number Diff line change
@@ -1,5 +1,5 @@
From mathcomp Require Import all_ssreflect ssralg ssrnum.
From mathcomp Require Import word_ssrZ.
From mathcomp Require Import ssreflect ssrfun ssrbool ssrnat eqtype finfun.
From mathcomp Require Import ssralg word_ssrZ.
Require oseq.
Require Import ZArith
utils
Expand Down
4 changes: 1 addition & 3 deletions proofs/arch/arch_utils.v
Original file line number Diff line number Diff line change
@@ -1,6 +1,4 @@
From mathcomp Require Import
all_ssreflect
ssralg ssrnum.
From mathcomp Require Import ssreflect ssrfun ssrbool ssrnat seq eqtype.

Require Import
type
Expand Down
3 changes: 1 addition & 2 deletions proofs/arch/asm_gen.v
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
From mathcomp Require Import all_ssreflect ssralg ssrnum.
From mathcomp Require Import ssreflect ssrfun ssrbool ssrnat eqtype ssralg.
Require Import
oseq
compiler_util
Expand All @@ -11,7 +11,6 @@ Require Import
arch_decl
arch_extra.
Import Utf8 String.
Import all_ssreflect.
Import compiler_util.

Set Implicit Arguments.
Expand Down
3 changes: 2 additions & 1 deletion proofs/arch/asm_gen_proof.v
Original file line number Diff line number Diff line change
@@ -1,4 +1,5 @@
From mathcomp Require Import all_ssreflect ssralg ssrnum.
From mathcomp Require Import ssreflect ssrfun ssrbool ssrnat eqtype.
From mathcomp Require Import fintype finfun ssralg.
From Coq Require Import Relation_Operators.
Require Import
oseq
Expand Down
2 changes: 1 addition & 1 deletion proofs/arch/label.v
Original file line number Diff line number Diff line change
@@ -1,5 +1,5 @@
(* -------------------------------------------------------------------- *)
From mathcomp Require Import all_ssreflect ssralg ssrnum.
From mathcomp Require Import ssreflect ssrfun ssrbool ssrnat eqtype ssralg.
Require Import global Utf8.

Set Implicit Arguments.
Expand Down
4 changes: 0 additions & 4 deletions proofs/arch/sem_params_of_arch_extra.v
Original file line number Diff line number Diff line change
@@ -1,7 +1,3 @@
From mathcomp Require Import
all_ssreflect
ssralg ssrnum.

Require Import
sem_params
syscall.
Expand Down
2 changes: 1 addition & 1 deletion proofs/compiler/allocation.v
Original file line number Diff line number Diff line change
@@ -1,5 +1,5 @@
(* ** Imports and settings *)
From mathcomp Require Import all_ssreflect ssralg ssrnum.
From mathcomp Require Import ssreflect ssrfun ssrbool ssrnat eqtype.
From mathcomp Require Import word_ssrZ.
Require Import expr compiler_util ZArith.
Import Utf8.
Expand Down
2 changes: 1 addition & 1 deletion proofs/compiler/allocation_proof.v
Original file line number Diff line number Diff line change
@@ -1,5 +1,5 @@
(* ** Imports and settings *)
From mathcomp Require Import all_ssreflect ssralg ssrnum.
From mathcomp Require Import ssreflect ssrfun ssrbool ssrnat eqtype.
Require Import psem compiler_util.
Require Export allocation.

Expand Down
1 change: 0 additions & 1 deletion proofs/compiler/arch_params.v
Original file line number Diff line number Diff line change
@@ -1,4 +1,3 @@
From mathcomp Require Import all_ssreflect ssralg ssrnum.
Require Import
compiler_util
expr.
Expand Down
3 changes: 1 addition & 2 deletions proofs/compiler/arch_params_proof.v
Original file line number Diff line number Diff line change
@@ -1,5 +1,4 @@

From mathcomp Require Import all_ssreflect ssralg ssrnum.
From mathcomp Require Import ssreflect ssrfun ssrbool ssrnat eqtype.
Require Import
compiler_util
expr
Expand Down
4 changes: 1 addition & 3 deletions proofs/compiler/arm.v
Original file line number Diff line number Diff line change
@@ -1,6 +1,4 @@
From mathcomp Require Import
all_ssreflect
ssralg ssrnum.
From mathcomp Require Import ssreflect ssrfun ssrbool eqtype.

Require Import utils.
Require Import arch_decl.
Expand Down
4 changes: 1 addition & 3 deletions proofs/compiler/arm_decl.v
Original file line number Diff line number Diff line change
@@ -1,6 +1,4 @@
From mathcomp Require Import
all_ssreflect
ssralg ssrnum.
From mathcomp Require Import ssreflect ssrfun ssrbool eqtype fintype ssralg.
From mathcomp Require Import word_ssrZ.

Require Import
Expand Down
4 changes: 1 addition & 3 deletions proofs/compiler/arm_extra.v
Original file line number Diff line number Diff line change
@@ -1,7 +1,5 @@
From HB Require Import structures.
From mathcomp Require Import
all_ssreflect
ssralg ssrnum.
From mathcomp Require Import ssreflect ssrfun ssrbool eqtype ssralg.

Require Import
compiler_util
Expand Down
4 changes: 1 addition & 3 deletions proofs/compiler/arm_facts.v
Original file line number Diff line number Diff line change
@@ -1,6 +1,4 @@
From mathcomp Require Import
all_ssreflect
ssralg ssrnum.
From mathcomp Require Import ssreflect ssrfun ssrbool eqtype ssralg.
From Coq Require Import ZArith.

Require Import
Expand Down
6 changes: 2 additions & 4 deletions proofs/compiler/arm_instr_decl.v
Original file line number Diff line number Diff line change
Expand Up @@ -3,10 +3,8 @@
These are the THUMB instructions of ARMv7-M, the instruction set of the M4
processor. *)

From mathcomp Require Import
all_ssreflect
ssralg ssrnum.
From mathcomp Require Import word_ssrZ.
From mathcomp Require Import ssreflect ssrfun ssrbool ssrnat seq eqtype fintype.
From mathcomp Require Import ssralg word_ssrZ.

Require Import
sem_type
Expand Down
4 changes: 1 addition & 3 deletions proofs/compiler/arm_instr_decl_lemmas.v
Original file line number Diff line number Diff line change
@@ -1,6 +1,4 @@
From mathcomp Require Import
all_ssreflect
ssralg ssrnum.
From mathcomp Require Import ssreflect ssrfun ssrbool.
From mathcomp Require Import word_ssrZ.

Require Import
Expand Down
4 changes: 1 addition & 3 deletions proofs/compiler/arm_lowering.v
Original file line number Diff line number Diff line change
@@ -1,6 +1,4 @@
From mathcomp Require Import
all_ssreflect
ssralg ssrnum.
From mathcomp Require Import ssreflect ssrfun ssrbool eqtype ssralg.
From mathcomp Require Import word_ssrZ.

Require Import
Expand Down
4 changes: 1 addition & 3 deletions proofs/compiler/arm_lowering_proof.v
Original file line number Diff line number Diff line change
@@ -1,6 +1,4 @@
From mathcomp Require Import
all_ssreflect
ssralg ssrnum.
From mathcomp Require Import ssreflect ssrfun ssrbool eqtype order ssralg.
Import
Order.POrderTheory
Order.TotalTheory.
Expand Down
5 changes: 1 addition & 4 deletions proofs/compiler/arm_params.v
Original file line number Diff line number Diff line change
@@ -1,7 +1,4 @@
From mathcomp Require Import
all_ssreflect
ssralg ssrnum.

From mathcomp Require Import ssreflect ssrfun ssrbool eqtype.
From mathcomp Require Import word_ssrZ.

Require Import
Expand Down
5 changes: 1 addition & 4 deletions proofs/compiler/arm_params_common.v
Original file line number Diff line number Diff line change
@@ -1,7 +1,4 @@
From mathcomp Require Import
all_ssreflect
ssralg ssrnum.

From mathcomp Require Import ssreflect ssrfun ssrbool.
From mathcomp Require Import word_ssrZ.

Require Import
Expand Down
5 changes: 1 addition & 4 deletions proofs/compiler/arm_params_common_proof.v
Original file line number Diff line number Diff line change
@@ -1,8 +1,5 @@
From Coq Require Import Lia.
From mathcomp Require Import
all_ssreflect
ssralg ssrnum.

From mathcomp Require Import ssreflect ssrfun ssrbool ssrnat eqtype ssralg.
From mathcomp Require Import word_ssrZ.

Require Import
Expand Down
5 changes: 1 addition & 4 deletions proofs/compiler/arm_params_core.v
Original file line number Diff line number Diff line change
@@ -1,7 +1,4 @@
From mathcomp Require Import
all_ssreflect
ssralg ssrnum.

From mathcomp Require Import ssreflect ssrfun ssrbool seq eqtype.
From mathcomp Require Import word_ssrZ.

Require Import
Expand Down
5 changes: 1 addition & 4 deletions proofs/compiler/arm_params_core_proof.v
Original file line number Diff line number Diff line change
@@ -1,8 +1,5 @@
From Coq Require Import Lia.
From mathcomp Require Import
all_ssreflect
ssralg ssrnum.

From mathcomp Require Import ssreflect ssrfun ssrbool ssrnat seq eqtype ssralg.
From mathcomp Require Import word_ssrZ.

Require Import
Expand Down
3 changes: 2 additions & 1 deletion proofs/compiler/arm_params_proof.v
Original file line number Diff line number Diff line change
@@ -1,5 +1,6 @@
From Coq Require Import Relations.
From mathcomp Require Import all_ssreflect ssralg ssrnum.
From mathcomp Require Import ssreflect ssrbool ssrfun eqtype ssrnat finfun.
From mathcomp Require Import ssralg.
From mathcomp Require Import word_ssrZ.

Require Import oseq.
Expand Down
2 changes: 1 addition & 1 deletion proofs/compiler/arm_stack_zeroization.v
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
From mathcomp Require Import all_ssreflect ssralg ssrnum.
From mathcomp Require Import ssreflect ssrfun ssrbool ssrnat eqtype.

Require Import
expr
Expand Down
2 changes: 1 addition & 1 deletion proofs/compiler/arm_stack_zeroization_proof.v
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
From mathcomp Require Import all_ssreflect ssralg ssrnum.
From mathcomp Require Import ssreflect ssrfun ssrbool ssrnat eqtype ssralg.
From mathcomp Require Import word_ssrZ.
Require Import Lia.

Expand Down
2 changes: 1 addition & 1 deletion proofs/compiler/array_copy.v
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
From mathcomp Require Import all_ssreflect.
From mathcomp Require Import ssreflect ssrfun ssrbool ssrnat eqtype.
Require Import
compiler_util
expr
Expand Down
2 changes: 1 addition & 1 deletion proofs/compiler/array_copy_proof.v
Original file line number Diff line number Diff line change
@@ -1,5 +1,5 @@
(* ** Imports and settings *)
From mathcomp Require Import all_ssreflect ssralg ssrnum.
From mathcomp Require Import ssreflect ssrfun ssrbool ssrnat eqtype.
From mathcomp Require Import word_ssrZ.
From Coq Require Import ZArith Lia.
Require Import array_copy psem.
Expand Down
2 changes: 1 addition & 1 deletion proofs/compiler/array_expansion.v
Original file line number Diff line number Diff line change
@@ -1,6 +1,6 @@
(* ** Imports and settings *)

From mathcomp Require Import all_ssreflect ssralg ssrnum.
From mathcomp Require Import ssreflect ssrfun ssrbool ssrnat eqtype.
From mathcomp Require Import word_ssrZ.
Require Import expr.
Require Import compiler_util ZArith.
Expand Down
2 changes: 1 addition & 1 deletion proofs/compiler/array_expansion_proof.v
Original file line number Diff line number Diff line change
@@ -1,5 +1,5 @@
(* ** Imports and settings *)
From mathcomp Require Import all_ssreflect ssralg ssrnum.
From mathcomp Require Import ssreflect ssrfun ssrbool ssrnat eqtype.
From mathcomp Require Import word_ssrZ.
Require Import psem array_expansion compiler_util ZArith.
Import Utf8 Lia.
Expand Down
2 changes: 1 addition & 1 deletion proofs/compiler/array_init.v
Original file line number Diff line number Diff line change
@@ -1,6 +1,6 @@
(* ** Imports and settings *)
Require Import ZArith.
From mathcomp Require Import all_ssreflect.
From mathcomp Require Import ssreflect ssrfun ssrbool.
Require Import expr compiler_util.

Set Implicit Arguments.
Expand Down
2 changes: 1 addition & 1 deletion proofs/compiler/array_init_proof.v
Original file line number Diff line number Diff line change
@@ -1,5 +1,5 @@
(* ** Imports and settings *)
From mathcomp Require Import all_ssreflect ssralg ssrnum.
From mathcomp Require Import ssreflect ssrfun ssrbool eqtype.
Require Import psem compiler_util.
Require Export array_init.
Import Utf8.
Expand Down
2 changes: 1 addition & 1 deletion proofs/compiler/byteset.v
Original file line number Diff line number Diff line change
@@ -1,6 +1,6 @@
(* ** Imports and settings *)
From HB Require Import structures.
From mathcomp Require Import all_ssreflect.
From mathcomp Require Import ssreflect ssrfun ssrbool ssrnat seq eqtype.
Require Import utils Wellfounded.
Import Lexicographic_Product Relation_Operators.

Expand Down
3 changes: 2 additions & 1 deletion proofs/compiler/compiler.v
Original file line number Diff line number Diff line change
@@ -1,5 +1,6 @@
From HB Require Import structures.
From mathcomp Require Import all_ssreflect ssralg ssrnum.
From mathcomp Require Import ssreflect ssrfun ssrbool ssrnat seq eqtype fintype.
From mathcomp Require Import ssralg.
Require Import ZArith.
Require Import Utf8.

Expand Down
3 changes: 2 additions & 1 deletion proofs/compiler/compiler_proof.v
Original file line number Diff line number Diff line change
@@ -1,4 +1,5 @@
From mathcomp Require Import all_ssreflect ssralg ssrnum.
From mathcomp Require Import ssreflect ssrfun ssrbool ssrnat seq eqtype.
From mathcomp Require Import fintype finfun ssralg.

Require Import
arch_params_proof
Expand Down
2 changes: 1 addition & 1 deletion proofs/compiler/compiler_util.v
Original file line number Diff line number Diff line change
@@ -1,5 +1,5 @@
Require Import ZArith Setoid Morphisms.
From mathcomp Require Import all_ssreflect ssralg ssrnum.
From mathcomp Require Import ssreflect ssrfun ssrbool ssrnat eqtype.
Require Import expr fexpr.

Set Implicit Arguments.
Expand Down
2 changes: 1 addition & 1 deletion proofs/compiler/constant_prop.v
Original file line number Diff line number Diff line change
@@ -1,8 +1,8 @@
(* ** Imports and settings *)
From HB Require Import structures.
From mathcomp Require Import ssreflect ssrfun ssrbool eqtype ssralg.
From mathcomp Require Import word_ssrZ.
Require Import expr ZArith sem_op_typed compiler_util.
Import all_ssreflect ssralg ssrnum.
Import Utf8.
Import oseq.
Require Import flag_combination.
Expand Down
2 changes: 1 addition & 1 deletion proofs/compiler/constant_prop_proof.v
Original file line number Diff line number Diff line change
@@ -1,5 +1,5 @@
(* ** Imports and settings *)
From mathcomp Require Import all_ssreflect ssralg ssrnum.
From mathcomp Require Import ssreflect ssrfun ssrbool ssrnat eqtype ssralg.
Require Import psem compiler_util.
Require Export constant_prop.

Expand Down
2 changes: 1 addition & 1 deletion proofs/compiler/dead_calls.v
Original file line number Diff line number Diff line change
@@ -1,5 +1,5 @@
(* -------------------------------------------------------------------- *)
From mathcomp Require Import all_ssreflect.
From mathcomp Require Import ssreflect ssrfun ssrbool.
(* ------- *) Require Import expr compiler_util gen_map.
(* ------- *) (* - *) Import PosSet.
Import Utf8.
Expand Down
2 changes: 1 addition & 1 deletion proofs/compiler/dead_calls_proof.v
Original file line number Diff line number Diff line change
@@ -1,5 +1,5 @@
(* -------------------------------------------------------------------- *)
From mathcomp Require Import all_ssreflect.
From mathcomp Require Import ssreflect ssrfun ssrbool eqtype.
(* ------- *) Require Import expr compiler_util psem gen_map dead_calls.
(* ------- *) (* - *) Import PosSet.
Import Utf8 xseq.
Expand Down
2 changes: 1 addition & 1 deletion proofs/compiler/dead_code.v
Original file line number Diff line number Diff line change
@@ -1,5 +1,5 @@
(* ** Imports and settings *)
From mathcomp Require Import all_ssreflect.
From mathcomp Require Import ssreflect ssrfun ssrbool eqtype.
Require Import expr compiler_util ZArith.

Set Implicit Arguments.
Expand Down
2 changes: 1 addition & 1 deletion proofs/compiler/dead_code_proof.v
Original file line number Diff line number Diff line change
@@ -1,5 +1,5 @@
(* ** Imports and settings *)
From mathcomp Require Import all_ssreflect ssralg ssrnum.
From mathcomp Require Import ssreflect ssrfun ssrbool eqtype.
Require Import psem compiler_util.
Require Export dead_code.
Import Utf8.
Expand Down
2 changes: 1 addition & 1 deletion proofs/compiler/direct_call_proof.v
Original file line number Diff line number Diff line change
@@ -1,5 +1,5 @@
(* ** Imports and settings *)
From mathcomp Require Import all_ssreflect ssralg ssrnum.
From mathcomp Require Import ssreflect ssrfun ssrbool.
Require Import varmap psem.

Import Utf8.
Expand Down
2 changes: 1 addition & 1 deletion proofs/compiler/inline.v
Original file line number Diff line number Diff line change
@@ -1,6 +1,6 @@
(* ** Imports and settings *)
Require Import ZArith.
From mathcomp Require Import all_ssreflect.
From mathcomp Require Import ssreflect ssrfun ssrbool.
Require Import expr compiler_util allocation.

Set Implicit Arguments.
Expand Down
2 changes: 1 addition & 1 deletion proofs/compiler/inline_proof.v
Original file line number Diff line number Diff line change
@@ -1,6 +1,6 @@
(* ** Imports and settings *)
Require Import ZArith.
From mathcomp Require Import all_ssreflect ssralg ssrnum.
From mathcomp Require Import ssreflect ssrfun ssrbool eqtype.
Require Import psem allocation_proof compiler_util.
Require Export inline.

Expand Down
2 changes: 1 addition & 1 deletion proofs/compiler/lea.v
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
From mathcomp Require Import all_ssreflect ssralg ssrnum.
From mathcomp Require Import ssreflect ssrfun ssrbool eqtype.
From mathcomp Require Import word_ssrZ.
Require Import Utf8.
Require Import expr.
Expand Down
2 changes: 1 addition & 1 deletion proofs/compiler/lea_proof.v
Original file line number Diff line number Diff line change
@@ -1,5 +1,5 @@
(* ** Imports and settings *)
From mathcomp Require Import all_ssreflect ssralg ssrnum.
From mathcomp Require Import ssreflect ssrfun ssrbool eqtype ssralg.
Require Import oseq.
Require Import psem compiler_util.
Require Import fexpr fexpr_sem fexpr_facts.
Expand Down
2 changes: 1 addition & 1 deletion proofs/compiler/linear_util.v
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
From mathcomp Require Import all_ssreflect ssralg ssrnum.
From mathcomp Require Import ssreflect ssrfun ssrbool eqtype.
Require Import expr label linear.
Require Import seq_extra compiler_util.

Expand Down
2 changes: 1 addition & 1 deletion proofs/compiler/linearization.v
Original file line number Diff line number Diff line change
Expand Up @@ -2,7 +2,7 @@

(* ** Imports and settings *)

From mathcomp Require Import all_ssreflect ssralg ssrnum.
From mathcomp Require Import ssreflect ssrfun ssrbool ssrnat seq eqtype.
Require Import ZArith.
Require Import Utf8.
Import Relations.
Expand Down
Loading

0 comments on commit cbad9fb

Please sign in to comment.