aboutsummaryrefslogtreecommitdiffhomepage
path: root/interp
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-06-22 06:31:30 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-06-22 06:31:30 +0000
commitd6c87f235a98c05a26b4a0e87129335d034219af (patch)
tree0cdbf9db7dc808621befc220892b9b7e083cdfe0 /interp
parenta1f06f016be512c21cb475491ec9924eea7ff288 (diff)
New script dev/tools/change-header to automatically update Coq files headers.
Applied it to fix mli file headers. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@13176 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'interp')
-rw-r--r--interp/constrextern.mli14
-rw-r--r--interp/constrintern.mli14
-rw-r--r--interp/coqlib.mli14
-rw-r--r--interp/dumpglob.mli14
-rw-r--r--interp/genarg.mli14
-rw-r--r--interp/implicit_quantifiers.mli14
-rw-r--r--interp/modintern.mli14
-rw-r--r--interp/notation.mli14
-rw-r--r--interp/ppextend.mli14
-rw-r--r--interp/reserve.mli14
-rw-r--r--interp/smartlocate.mli14
-rw-r--r--interp/syntax_def.mli14
-rw-r--r--interp/topconstr.mli14
13 files changed, 91 insertions, 91 deletions
diff --git a/interp/constrextern.mli b/interp/constrextern.mli
index ac3a38833..7bc2ddcec 100644
--- a/interp/constrextern.mli
+++ b/interp/constrextern.mli
@@ -1,10 +1,10 @@
-(***********************************************************************
- v * The Coq Proof Assistant / The Coq Development Team
- <O___,, * CNRS-Ecole Polytechnique-INRIA Futurs-Universite Paris Sud
- \VV/ *************************************************************
- // * This file is distributed under the terms of the
- * GNU Lesser General Public License Version 2.1
- ***********************************************************************)
+(************************************************************************)
+(* v * The Coq Proof Assistant / The Coq Development Team *)
+(* <O___,, * CNRS-Ecole Polytechnique-INRIA Futurs-Universite Paris Sud *)
+(* \VV/ **************************************************************)
+(* // * This file is distributed under the terms of the *)
+(* * GNU Lesser General Public License Version 2.1 *)
+(************************************************************************)
open Util
open Names
diff --git a/interp/constrintern.mli b/interp/constrintern.mli
index 880f8a4be..62821081f 100644
--- a/interp/constrintern.mli
+++ b/interp/constrintern.mli
@@ -1,10 +1,10 @@
-(***********************************************************************
- v * The Coq Proof Assistant / The Coq Development Team
- <O___,, * CNRS-Ecole Polytechnique-INRIA Futurs-Universite Paris Sud
- \VV/ *************************************************************
- // * This file is distributed under the terms of the
- * GNU Lesser General Public License Version 2.1
- ***********************************************************************)
+(************************************************************************)
+(* v * The Coq Proof Assistant / The Coq Development Team *)
+(* <O___,, * CNRS-Ecole Polytechnique-INRIA Futurs-Universite Paris Sud *)
+(* \VV/ **************************************************************)
+(* // * This file is distributed under the terms of the *)
+(* * GNU Lesser General Public License Version 2.1 *)
+(************************************************************************)
open Names
open Term
diff --git a/interp/coqlib.mli b/interp/coqlib.mli
index 1d7f571b3..73427d902 100644
--- a/interp/coqlib.mli
+++ b/interp/coqlib.mli
@@ -1,10 +1,10 @@
-(***********************************************************************
- v * The Coq Proof Assistant / The Coq Development Team
- <O___,, * CNRS-Ecole Polytechnique-INRIA Futurs-Universite Paris Sud
- \VV/ *************************************************************
- // * This file is distributed under the terms of the
- * GNU Lesser General Public License Version 2.1
- ***********************************************************************)
+(************************************************************************)
+(* v * The Coq Proof Assistant / The Coq Development Team *)
+(* <O___,, * CNRS-Ecole Polytechnique-INRIA Futurs-Universite Paris Sud *)
+(* \VV/ **************************************************************)
+(* // * This file is distributed under the terms of the *)
+(* * GNU Lesser General Public License Version 2.1 *)
+(************************************************************************)
open Names
open Libnames
diff --git a/interp/dumpglob.mli b/interp/dumpglob.mli
index 7efa6f1e0..023608490 100644
--- a/interp/dumpglob.mli
+++ b/interp/dumpglob.mli
@@ -1,10 +1,10 @@
-(***********************************************************************
- v * The Coq Proof Assistant / The Coq Development Team
- <O___,, * CNRS-Ecole Polytechnique-INRIA Futurs-Universite Paris Sud
- \VV/ *************************************************************
- // * This file is distributed under the terms of the
- * GNU Lesser General Public License Version 2.1
- ***********************************************************************)
+(************************************************************************)
+(* v * The Coq Proof Assistant / The Coq Development Team *)
+(* <O___,, * CNRS-Ecole Polytechnique-INRIA Futurs-Universite Paris Sud *)
+(* \VV/ **************************************************************)
+(* // * This file is distributed under the terms of the *)
+(* * GNU Lesser General Public License Version 2.1 *)
+(************************************************************************)
val open_glob_file : string -> unit
val close_glob_file : unit -> unit
diff --git a/interp/genarg.mli b/interp/genarg.mli
index 984f479fb..0ab3b4320 100644
--- a/interp/genarg.mli
+++ b/interp/genarg.mli
@@ -1,10 +1,10 @@
-(***********************************************************************
- v * The Coq Proof Assistant / The Coq Development Team
- <O___,, * CNRS-Ecole Polytechnique-INRIA Futurs-Universite Paris Sud
- \VV/ *************************************************************
- // * This file is distributed under the terms of the
- * GNU Lesser General Public License Version 2.1
- ***********************************************************************)
+(************************************************************************)
+(* v * The Coq Proof Assistant / The Coq Development Team *)
+(* <O___,, * CNRS-Ecole Polytechnique-INRIA Futurs-Universite Paris Sud *)
+(* \VV/ **************************************************************)
+(* // * This file is distributed under the terms of the *)
+(* * GNU Lesser General Public License Version 2.1 *)
+(************************************************************************)
open Util
open Names
diff --git a/interp/implicit_quantifiers.mli b/interp/implicit_quantifiers.mli
index 0b2ac3e71..cf3989f89 100644
--- a/interp/implicit_quantifiers.mli
+++ b/interp/implicit_quantifiers.mli
@@ -1,10 +1,10 @@
-(***********************************************************************
- v * The Coq Proof Assistant / The Coq Development Team
- <O___,, * CNRS-Ecole Polytechnique-INRIA Futurs-Universite Paris Sud
- \VV/ *************************************************************
- // * This file is distributed under the terms of the
- * GNU Lesser General Public License Version 2.1
- ***********************************************************************)
+(************************************************************************)
+(* v * The Coq Proof Assistant / The Coq Development Team *)
+(* <O___,, * CNRS-Ecole Polytechnique-INRIA Futurs-Universite Paris Sud *)
+(* \VV/ **************************************************************)
+(* // * This file is distributed under the terms of the *)
+(* * GNU Lesser General Public License Version 2.1 *)
+(************************************************************************)
open Names
open Decl_kinds
diff --git a/interp/modintern.mli b/interp/modintern.mli
index 5dacfd070..c5940bfff 100644
--- a/interp/modintern.mli
+++ b/interp/modintern.mli
@@ -1,10 +1,10 @@
-(***********************************************************************
- v * The Coq Proof Assistant / The Coq Development Team
- <O___,, * CNRS-Ecole Polytechnique-INRIA Futurs-Universite Paris Sud
- \VV/ *************************************************************
- // * This file is distributed under the terms of the
- * GNU Lesser General Public License Version 2.1
- ***********************************************************************)
+(************************************************************************)
+(* v * The Coq Proof Assistant / The Coq Development Team *)
+(* <O___,, * CNRS-Ecole Polytechnique-INRIA Futurs-Universite Paris Sud *)
+(* \VV/ **************************************************************)
+(* // * This file is distributed under the terms of the *)
+(* * GNU Lesser General Public License Version 2.1 *)
+(************************************************************************)
open Declarations
open Environ
diff --git a/interp/notation.mli b/interp/notation.mli
index 3da9ec0e5..17d8ad8f2 100644
--- a/interp/notation.mli
+++ b/interp/notation.mli
@@ -1,10 +1,10 @@
-(***********************************************************************
- v * The Coq Proof Assistant / The Coq Development Team
- <O___,, * CNRS-Ecole Polytechnique-INRIA Futurs-Universite Paris Sud
- \VV/ *************************************************************
- // * This file is distributed under the terms of the
- * GNU Lesser General Public License Version 2.1
- ***********************************************************************)
+(************************************************************************)
+(* v * The Coq Proof Assistant / The Coq Development Team *)
+(* <O___,, * CNRS-Ecole Polytechnique-INRIA Futurs-Universite Paris Sud *)
+(* \VV/ **************************************************************)
+(* // * This file is distributed under the terms of the *)
+(* * GNU Lesser General Public License Version 2.1 *)
+(************************************************************************)
open Util
open Pp
diff --git a/interp/ppextend.mli b/interp/ppextend.mli
index 19ca913e8..99152c045 100644
--- a/interp/ppextend.mli
+++ b/interp/ppextend.mli
@@ -1,10 +1,10 @@
-(***********************************************************************
- v * The Coq Proof Assistant / The Coq Development Team
- <O___,, * CNRS-Ecole Polytechnique-INRIA Futurs-Universite Paris Sud
- \VV/ *************************************************************
- // * This file is distributed under the terms of the
- * GNU Lesser General Public License Version 2.1
- ***********************************************************************)
+(************************************************************************)
+(* v * The Coq Proof Assistant / The Coq Development Team *)
+(* <O___,, * CNRS-Ecole Polytechnique-INRIA Futurs-Universite Paris Sud *)
+(* \VV/ **************************************************************)
+(* // * This file is distributed under the terms of the *)
+(* * GNU Lesser General Public License Version 2.1 *)
+(************************************************************************)
open Pp
open Names
diff --git a/interp/reserve.mli b/interp/reserve.mli
index e53ad8365..184eb2183 100644
--- a/interp/reserve.mli
+++ b/interp/reserve.mli
@@ -1,10 +1,10 @@
-(***********************************************************************
- v * The Coq Proof Assistant / The Coq Development Team
- <O___,, * CNRS-Ecole Polytechnique-INRIA Futurs-Universite Paris Sud
- \VV/ *************************************************************
- // * This file is distributed under the terms of the
- * GNU Lesser General Public License Version 2.1
- ***********************************************************************)
+(************************************************************************)
+(* v * The Coq Proof Assistant / The Coq Development Team *)
+(* <O___,, * CNRS-Ecole Polytechnique-INRIA Futurs-Universite Paris Sud *)
+(* \VV/ **************************************************************)
+(* // * This file is distributed under the terms of the *)
+(* * GNU Lesser General Public License Version 2.1 *)
+(************************************************************************)
open Util
open Names
diff --git a/interp/smartlocate.mli b/interp/smartlocate.mli
index 0cd261a82..b5a89949f 100644
--- a/interp/smartlocate.mli
+++ b/interp/smartlocate.mli
@@ -1,10 +1,10 @@
-(***********************************************************************
- v * The Coq Proof Assistant / The Coq Development Team
- <O___,, * CNRS-Ecole Polytechnique-INRIA Futurs-Universite Paris Sud
- \VV/ *************************************************************
- // * This file is distributed under the terms of the
- * GNU Lesser General Public License Version 2.1
- ***********************************************************************)
+(************************************************************************)
+(* v * The Coq Proof Assistant / The Coq Development Team *)
+(* <O___,, * CNRS-Ecole Polytechnique-INRIA Futurs-Universite Paris Sud *)
+(* \VV/ **************************************************************)
+(* // * This file is distributed under the terms of the *)
+(* * GNU Lesser General Public License Version 2.1 *)
+(************************************************************************)
open Util
open Names
diff --git a/interp/syntax_def.mli b/interp/syntax_def.mli
index 019067608..94252950b 100644
--- a/interp/syntax_def.mli
+++ b/interp/syntax_def.mli
@@ -1,10 +1,10 @@
-(***********************************************************************
- v * The Coq Proof Assistant / The Coq Development Team
- <O___,, * CNRS-Ecole Polytechnique-INRIA Futurs-Universite Paris Sud
- \VV/ *************************************************************
- // * This file is distributed under the terms of the
- * GNU Lesser General Public License Version 2.1
- ***********************************************************************)
+(************************************************************************)
+(* v * The Coq Proof Assistant / The Coq Development Team *)
+(* <O___,, * CNRS-Ecole Polytechnique-INRIA Futurs-Universite Paris Sud *)
+(* \VV/ **************************************************************)
+(* // * This file is distributed under the terms of the *)
+(* * GNU Lesser General Public License Version 2.1 *)
+(************************************************************************)
open Util
open Names
diff --git a/interp/topconstr.mli b/interp/topconstr.mli
index b288fe8b5..3a50475db 100644
--- a/interp/topconstr.mli
+++ b/interp/topconstr.mli
@@ -1,10 +1,10 @@
-(***********************************************************************
- v * The Coq Proof Assistant / The Coq Development Team
- <O___,, * CNRS-Ecole Polytechnique-INRIA Futurs-Universite Paris Sud
- \VV/ *************************************************************
- // * This file is distributed under the terms of the
- * GNU Lesser General Public License Version 2.1
- ***********************************************************************)
+(************************************************************************)
+(* v * The Coq Proof Assistant / The Coq Development Team *)
+(* <O___,, * CNRS-Ecole Polytechnique-INRIA Futurs-Universite Paris Sud *)
+(* \VV/ **************************************************************)
+(* // * This file is distributed under the terms of the *)
+(* * GNU Lesser General Public License Version 2.1 *)
+(************************************************************************)
open Pp
open Util