aboutsummaryrefslogtreecommitdiff
path: root/mathcomp/character/mxabelem.v
diff options
context:
space:
mode:
authorCyril Cohen2015-04-09 16:13:05 +0200
committerCyril Cohen2015-04-09 16:13:05 +0200
commitf180c539a00fd83d8b3b5fd2d5710eb16e971e2e (patch)
tree778f055ca9eaba4fe8991f9099cb436483cad943 /mathcomp/character/mxabelem.v
parent2a8980122824511b3356b09b88a7f152427f2df6 (diff)
character for v8.5
Diffstat (limited to 'mathcomp/character/mxabelem.v')
-rw-r--r--mathcomp/character/mxabelem.v17
1 files changed, 13 insertions, 4 deletions
diff --git a/mathcomp/character/mxabelem.v b/mathcomp/character/mxabelem.v
index 188000d..377cb72 100644
--- a/mathcomp/character/mxabelem.v
+++ b/mathcomp/character/mxabelem.v
@@ -1,9 +1,18 @@
(* (c) Copyright Microsoft Corporation and Inria. All rights reserved. *)
-Require Import ssreflect ssrbool ssrfun eqtype ssrnat seq path div choice.
-Require Import fintype tuple finfun bigop prime ssralg poly finset.
+Require Import mathcomp.ssreflect.ssreflect.
+From mathcomp.ssreflect
+Require Import ssreflect ssrbool ssrfun eqtype ssrnat seq.
+From mathcomp.discrete
+Require Import path div choice fintype tuple finfun bigop prime finset.
+From mathcomp.fingroup
Require Import fingroup morphism perm automorphism quotient gproduct action.
-Require Import finalg zmodp commutator cyclic center pgroup gseries nilpotent.
-Require Import sylow maximal abelian matrix mxalgebra mxrepresentation.
+From mathcomp.algebra
+Require Import ssralg poly finalg zmodp cyclic matrix mxalgebra.
+From mathcomp.solvable
+Require Import commutator center pgroup gseries nilpotent.
+From mathcomp.solvable
+Require Import sylow maximal abelian.
+Require Import mxrepresentation.
(******************************************************************************)
(* This file completes the theory developed in mxrepresentation.v with the *)