Skip to content

Commit

Permalink
prepared discrete for compilation in v8.5
Browse files Browse the repository at this point in the history
  • Loading branch information
CohenCyril committed Apr 3, 2015
1 parent 9859058 commit 9fa572c
Show file tree
Hide file tree
Showing 13 changed files with 30 additions and 15 deletions.
1 change: 0 additions & 1 deletion mathcomp/discrete/all.v
Original file line number Diff line number Diff line change
@@ -1,4 +1,3 @@
Require Export mathcomp.ssreflect.all.
Require Export choice.
Require Export path.
Require Export div.
Expand Down
5 changes: 3 additions & 2 deletions mathcomp/discrete/bigop.v
Original file line number Diff line number Diff line change
@@ -1,6 +1,7 @@
(* (c) Copyright Microsoft Corporation and Inria. All rights reserved. *)
Require Import ssreflect ssrbool ssrfun eqtype ssrnat seq path div fintype.
Require Import tuple finfun.
(*v8.5 From mathcomp.ssreflect *)
Require Import ssreflect ssrbool ssrfun eqtype ssrnat seq.
Require Import path div fintype tuple finfun.

(******************************************************************************)
(* This file provides a generic definition for iterating an operator over a *)
Expand Down
5 changes: 3 additions & 2 deletions mathcomp/discrete/binomial.v
Original file line number Diff line number Diff line change
@@ -1,6 +1,7 @@
(* (c) Copyright Microsoft Corporation and Inria. All rights reserved. *)
Require Import ssreflect ssrfun ssrbool eqtype ssrnat seq path div.
Require Import fintype tuple finfun bigop prime finset.
(*v8.5 From mathcomp.ssreflect *)
Require Import ssreflect ssrfun ssrbool eqtype ssrnat seq.
Require Import path div fintype tuple finfun bigop prime finset.

(******************************************************************************)
(* This files contains the definition of: *)
Expand Down
1 change: 1 addition & 0 deletions mathcomp/discrete/choice.v
Original file line number Diff line number Diff line change
@@ -1,4 +1,5 @@
(* (c) Copyright Microsoft Corporation and Inria. All rights reserved. *)
(*v8.5 From mathcomp.ssreflect *)
Require Import ssreflect ssrfun ssrbool eqtype ssrnat seq.

(******************************************************************************)
Expand Down
1 change: 1 addition & 0 deletions mathcomp/discrete/div.v
Original file line number Diff line number Diff line change
@@ -1,4 +1,5 @@
(* (c) Copyright Microsoft Corporation and Inria. All rights reserved. *)
(*v8.5 From mathcomp.ssreflect *)
Require Import ssreflect ssrfun ssrbool eqtype ssrnat seq.

(******************************************************************************)
Expand Down
4 changes: 3 additions & 1 deletion mathcomp/discrete/finfun.v
Original file line number Diff line number Diff line change
@@ -1,5 +1,7 @@
(* (c) Copyright Microsoft Corporation and Inria. All rights reserved. *)
Require Import ssreflect ssrfun ssrbool eqtype ssrnat seq choice fintype tuple.
(*v8.5 From mathcomp.ssreflect *)
Require Import ssreflect ssrfun ssrbool eqtype ssrnat seq.
Require Import choice fintype tuple.

(******************************************************************************)
(* This file implements a type for functions with a finite domain: *)
Expand Down
4 changes: 3 additions & 1 deletion mathcomp/discrete/fingraph.v
Original file line number Diff line number Diff line change
@@ -1,5 +1,7 @@
(* (c) Copyright Microsoft Corporation and Inria. All rights reserved. *)
Require Import ssreflect ssrbool ssrfun eqtype ssrnat seq path fintype.
(*v8.5 From mathcomp.ssreflect *)
Require Import ssreflect ssrbool ssrfun eqtype ssrnat seq.
Require Import path fintype.

(******************************************************************************)
(* This file develops the theory of finite graphs represented by an "edge" *)
Expand Down
5 changes: 3 additions & 2 deletions mathcomp/discrete/finset.v
Original file line number Diff line number Diff line change
@@ -1,6 +1,7 @@
(* (c) Copyright Microsoft Corporation and Inria. All rights reserved. *)
Require Import ssreflect ssrbool ssrfun eqtype ssrnat div seq choice fintype.
Require Import finfun bigop.
(*v8.5 From mathcomp.ssreflect *)
Require Import ssreflect ssrbool ssrfun eqtype ssrnat seq.
Require Import bigop choice fintype div finfun.

(******************************************************************************)
(* This file defines a type for sets over a finite Type, similar to the type *)
Expand Down
4 changes: 3 additions & 1 deletion mathcomp/discrete/fintype.v
Original file line number Diff line number Diff line change
@@ -1,5 +1,7 @@
(* (c) Copyright Microsoft Corporation and Inria. All rights reserved. *)
Require Import ssreflect ssrfun ssrbool eqtype ssrnat seq choice.
(*v8.5 From mathcomp.ssreflect *)
Require Import ssreflect ssrfun ssrbool eqtype ssrnat seq.
Require Import choice.

(******************************************************************************)
(* The Finite interface describes Types with finitely many elements, *)
Expand Down
5 changes: 3 additions & 2 deletions mathcomp/discrete/generic_quotient.v
Original file line number Diff line number Diff line change
@@ -1,7 +1,8 @@
(* (c) Copyright Microsoft Corporation and Inria. All rights reserved. *)
(* -*- coding : utf-8 -*- *)

Require Import ssreflect ssrfun ssrbool eqtype ssrnat choice seq fintype.
(*v8.5 From mathcomp.ssreflect *)
Require Import ssreflect ssrfun ssrbool eqtype ssrnat seq.
Require Import choice fintype.

(*****************************************************************************)
(* Provided a base type T, this files defines an interface for quotients Q *)
Expand Down
1 change: 1 addition & 0 deletions mathcomp/discrete/path.v
Original file line number Diff line number Diff line change
@@ -1,4 +1,5 @@
(* (c) Copyright Microsoft Corporation and Inria. All rights reserved. *)
(*v8.5 From mathcomp.ssreflect *)
Require Import ssreflect ssrfun ssrbool eqtype ssrnat seq.

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

(******************************************************************************)
(* This file contains the definitions of: *)
Expand Down
4 changes: 3 additions & 1 deletion mathcomp/discrete/tuple.v
Original file line number Diff line number Diff line change
@@ -1,5 +1,7 @@
(* (c) Copyright Microsoft Corporation and Inria. All rights reserved. *)
Require Import ssreflect ssrfun ssrbool eqtype ssrnat seq choice fintype.
(*v8.5 From mathcomp.ssreflect *)
Require Import ssreflect ssrfun ssrbool eqtype ssrnat seq.
Require Import choice fintype.

Set Implicit Arguments.
Unset Strict Implicit.
Expand Down

0 comments on commit 9fa572c

Please sign in to comment.