aboutsummaryrefslogtreecommitdiff
path: root/mathcomp/algebra/mxpoly.v
diff options
context:
space:
mode:
authorCyril Cohen2015-04-08 15:36:17 +0200
committerCyril Cohen2015-04-08 15:36:17 +0200
commitde1794e797c69ffa8f878c3e8b6f0fb2b6ec5ef5 (patch)
treec2c1e064e50e44c64e390f750c92e3204f2791ae /mathcomp/algebra/mxpoly.v
parent858957ad3a4e3cfdd98fd5c9f172b564d6871442 (diff)
packaging for v8.5
Diffstat (limited to 'mathcomp/algebra/mxpoly.v')
-rw-r--r--mathcomp/algebra/mxpoly.v10
1 files changed, 7 insertions, 3 deletions
diff --git a/mathcomp/algebra/mxpoly.v b/mathcomp/algebra/mxpoly.v
index 7e889a0..8a0b519 100644
--- a/mathcomp/algebra/mxpoly.v
+++ b/mathcomp/algebra/mxpoly.v
@@ -1,7 +1,11 @@
(* (c) Copyright Microsoft Corporation and Inria. All rights reserved. *)
-Require Import ssreflect ssrfun ssrbool eqtype ssrnat seq div fintype tuple.
-Require Import finfun bigop fingroup perm ssralg zmodp matrix mxalgebra.
-Require Import poly polydiv.
+(*v8.5 From mathcomp.ssreflect *)
+Require Import ssreflect ssrfun ssrbool eqtype ssrnat seq.
+(*v8.5 From mathcomp.discrete *)
+Require Import div fintype tuple finfun bigop.
+(*v8.5 From mathcomp.fingroup *)
+Require Import fingroup perm.
+Require Import ssralg zmodp matrix mxalgebra poly polydiv.
(******************************************************************************)
(* This file provides basic support for formal computation with matrices, *)