Skip to content

Commit

Permalink
packaging for v8.5
Browse files Browse the repository at this point in the history
  • Loading branch information
CohenCyril committed Apr 8, 2015
1 parent 737f79e commit 858957a
Show file tree
Hide file tree
Showing 8 changed files with 37 additions and 14 deletions.
7 changes: 5 additions & 2 deletions mathcomp/fingroup/action.v
Original file line number Diff line number Diff line change
@@ -1,6 +1,9 @@
(* (c) Copyright Microsoft Corporation and Inria. All rights reserved. *)
Require Import ssreflect ssrbool ssrfun eqtype ssrnat div seq fintype.
Require Import bigop finset fingroup morphism perm automorphism quotient.
(*v8.5 From mathcomp.ssreflect *)
Require Import ssreflect ssrbool ssrfun eqtype ssrnat seq.
(*v8.5 From mathcomp.discrete *)
Require Import div fintype bigop finset.
Require Import fingroup morphism perm automorphism quotient.

(******************************************************************************)
(* Group action: orbits, stabilisers, transitivity. *)
Expand Down
5 changes: 4 additions & 1 deletion mathcomp/fingroup/automorphism.v
Original file line number Diff line number Diff line change
@@ -1,5 +1,8 @@
(* (c) Copyright Microsoft Corporation and Inria. All rights reserved. *)
Require Import ssreflect ssrbool ssrfun eqtype ssrnat fintype finset.
(*v8.5 From mathcomp.ssreflect *)
Require Import ssreflect ssrbool ssrfun eqtype ssrnat.
(*v8.5 From mathcomp.discrete *)
Require Import fintype finset.
Require Import fingroup perm morphism.

(******************************************************************************)
Expand Down
6 changes: 4 additions & 2 deletions mathcomp/fingroup/fingroup.v
Original file line number Diff line number Diff line change
@@ -1,6 +1,8 @@
(* (c) Copyright Microsoft Corporation and Inria. All rights reserved. *)
Require Import ssreflect ssrbool ssrfun eqtype ssrnat seq choice fintype.
Require Import div path bigop prime finset.
(*v8.5 From mathcomp.ssreflect *)
Require Import ssreflect ssrbool ssrfun eqtype ssrnat seq.
(*v8.5 From mathcomp.discrete *)
Require Import choice fintype div path bigop prime finset.

(******************************************************************************)
(* This file defines the main interface for finite groups : *)
Expand Down
7 changes: 5 additions & 2 deletions mathcomp/fingroup/gproduct.v
Original file line number Diff line number Diff line change
@@ -1,6 +1,9 @@
(* (c) Copyright Microsoft Corporation and Inria. All rights reserved. *)
Require Import ssreflect ssrbool ssrfun eqtype ssrnat seq div choice fintype.
Require Import bigop finset fingroup morphism quotient action.
(*v8.5 From mathcomp.ssreflect *)
Require Import ssreflect ssrbool ssrfun eqtype ssrnat seq.
(*v8.5 From mathcomp.discrete *)
Require Import div choice fintype bigop finset.
Require Import fingroup morphism quotient action.

(******************************************************************************)
(* Partial, semidirect, central, and direct products. *)
Expand Down
7 changes: 5 additions & 2 deletions mathcomp/fingroup/morphism.v
Original file line number Diff line number Diff line change
@@ -1,6 +1,9 @@
(* (c) Copyright Microsoft Corporation and Inria. All rights reserved. *)
Require Import ssreflect ssrbool ssrfun eqtype ssrnat seq choice fintype finfun.
Require Import bigop finset fingroup.
(*v8.5 From mathcomp.ssreflect *)
Require Import ssreflect ssrbool ssrfun eqtype ssrnat seq.
(*v8.5 From mathcomp.discrete *)
Require Import choice fintype finfun bigop finset.
Require Import fingroup.

(******************************************************************************)
(* This file contains the definitions of: *)
Expand Down
7 changes: 5 additions & 2 deletions mathcomp/fingroup/perm.v
Original file line number Diff line number Diff line change
@@ -1,6 +1,9 @@
(* (c) Copyright Microsoft Corporation and Inria. All rights reserved. *)
Require Import ssreflect ssrfun ssrbool eqtype ssrnat seq path choice fintype.
Require Import tuple finfun bigop finset binomial fingroup.
(*v8.5 From mathcomp.ssreflect *)
Require Import ssreflect ssrfun ssrbool eqtype ssrnat seq.
(*v8.5 From mathcomp.discrete *)
Require Import path choice fintype tuple finfun bigop finset binomial.
Require Import fingroup.

(******************************************************************************)
(* This file contains the definition and properties associated to the group *)
Expand Down
5 changes: 4 additions & 1 deletion mathcomp/fingroup/presentation.v
Original file line number Diff line number Diff line change
@@ -1,5 +1,8 @@
(* (c) Copyright Microsoft Corporation and Inria. All rights reserved. *)
Require Import ssreflect ssrbool ssrfun eqtype ssrnat seq fintype finset.
(*v8.5 From mathcomp.ssreflect *)
Require Import ssreflect ssrbool ssrfun eqtype ssrnat seq.
(*v8.5 From mathcomp.discrete *)
Require Import fintype finset.
Require Import fingroup morphism.

(******************************************************************************)
Expand Down
7 changes: 5 additions & 2 deletions mathcomp/fingroup/quotient.v
Original file line number Diff line number Diff line change
@@ -1,6 +1,9 @@
(* (c) Copyright Microsoft Corporation and Inria. All rights reserved. *)
Require Import ssreflect ssrfun ssrbool eqtype ssrnat seq div choice.
Require Import fintype prime finset fingroup morphism automorphism.
(*v8.5 From mathcomp.ssreflect *)
Require Import ssreflect ssrfun ssrbool eqtype ssrnat seq.
(*v8.5 From mathcomp.discrete *)
Require Import div choice fintype prime finset.
Require Import fingroup morphism automorphism.

(******************************************************************************)
(* This file contains the definitions of: *)
Expand Down

0 comments on commit 858957a

Please sign in to comment.