Skip to content

Commit

Permalink
Makefile, testing for v8.5 and uncommenting stuff
Browse files Browse the repository at this point in the history
This is a temporary solution, but there is a better one :
one could patch ssreflect.ml4 plugin for v8.4 to interpret
From ... Require Import ... as a simple Require Import.
  • Loading branch information
CohenCyril committed Apr 3, 2015
1 parent 9fa572c commit abe2354
Show file tree
Hide file tree
Showing 13 changed files with 19 additions and 12 deletions.
7 changes: 7 additions & 0 deletions mathcomp/discrete/Makefile
Original file line number Diff line number Diff line change
Expand Up @@ -5,12 +5,19 @@ COQBIN=$(dir $(shell which coqtop))/
endif


VERSION_Coq = $(shell $(COQBIN)/coqtop -v | head -1 | sed 's/.*version \([0-9]\.[0-9]\)[^ ]* .*/v\1/')

ifeq "$(VERSION_Coq)" ""
$(error no version number found for coq)
endif

OLD_MAKEFLAGS:=$(MAKEFLAGS)
MAKEFLAGS+=-B

.DEFAULT_GOAL := all

%:
sed -i -e "s/^(\*$(VERSION_Coq) *\(.*\) *\*)/\1/" *.v
$(H)[ -e Makefile.coq ] || $(COQBIN)/coq_makefile -f Make -o Makefile.coq
$(H)MAKEFLAGS=$(OLD_MAKEFLAGS) $(MAKE) --no-print-directory \
-f Makefile.coq $*
Expand Down
2 changes: 1 addition & 1 deletion mathcomp/discrete/bigop.v
Original file line number Diff line number Diff line change
@@ -1,5 +1,5 @@
(* (c) Copyright Microsoft Corporation and Inria. All rights reserved. *)
(*v8.5 From mathcomp.ssreflect *)
(*v8.5 From mathcomp.ssreflect *)
Require Import ssreflect ssrbool ssrfun eqtype ssrnat seq.
Require Import path div fintype tuple finfun.

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

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

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

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

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

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

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

Expand Down
2 changes: 1 addition & 1 deletion mathcomp/discrete/generic_quotient.v
Original file line number Diff line number Diff line change
@@ -1,6 +1,6 @@
(* (c) Copyright Microsoft Corporation and Inria. All rights reserved. *)
(* -*- coding : utf-8 -*- *)
(*v8.5 From mathcomp.ssreflect *)
(*v8.5 From mathcomp.ssreflect *)
Require Import ssreflect ssrfun ssrbool eqtype ssrnat seq.
Require Import choice fintype.

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

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

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

Expand Down

0 comments on commit abe2354

Please sign in to comment.