aboutsummaryrefslogtreecommitdiff
path: root/mathcomp/algebra/vector.v
diff options
context:
space:
mode:
authorGeorges Gonthier2019-04-28 11:31:11 +0200
committerGitHub2019-04-28 11:31:11 +0200
commit8e27a1dd704c8f7a34de29d65337eb67254a1741 (patch)
tree240ce34774221645650404da1337e94c5e3f63b3 /mathcomp/algebra/vector.v
parentdec1f90d13c44016ea53da360e9692fd768bc24b (diff)
parent22c182b681c2852afa13efc2bc1d6d083646f061 (diff)
Merge pull request #336 from CohenCyril/clean_require
Cleaning Require and Require Imports
Diffstat (limited to 'mathcomp/algebra/vector.v')
-rw-r--r--mathcomp/algebra/vector.v8
1 files changed, 3 insertions, 5 deletions
diff --git a/mathcomp/algebra/vector.v b/mathcomp/algebra/vector.v
index 4766c74..48d7d3e 100644
--- a/mathcomp/algebra/vector.v
+++ b/mathcomp/algebra/vector.v
@@ -1,10 +1,8 @@
(* (c) Copyright 2006-2016 Microsoft Corporation and Inria. *)
(* Distributed under the terms of CeCILL-B. *)
-Require Import mathcomp.ssreflect.ssreflect.
-From mathcomp
-Require Import ssrfun ssrbool eqtype ssrnat seq choice fintype bigop.
-From mathcomp
-Require Import finfun tuple ssralg matrix mxalgebra zmodp.
+From mathcomp Require Import ssreflect ssrfun ssrbool eqtype ssrnat seq choice.
+From mathcomp Require Import fintype bigop finfun tuple.
+From mathcomp Require Import ssralg matrix mxalgebra zmodp.
(******************************************************************************)
(* * Finite dimensional vector spaces *)