aboutsummaryrefslogtreecommitdiffhomepage
path: root/lib
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 /lib
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 'lib')
-rw-r--r--lib/bigint.mli14
-rw-r--r--lib/dnet.mli14
-rw-r--r--lib/dyn.mli14
-rw-r--r--lib/envars.mli14
-rw-r--r--lib/explore.mli14
-rw-r--r--lib/flags.mli14
-rw-r--r--lib/gmap.mli14
-rw-r--r--lib/gmapl.mli14
-rw-r--r--lib/gset.mli14
-rw-r--r--lib/hashcons.mli14
-rw-r--r--lib/heap.mli14
-rw-r--r--lib/option.mli14
-rw-r--r--lib/pp.mli14
-rw-r--r--lib/pp_control.mli14
-rw-r--r--lib/profile.mli14
-rw-r--r--lib/rtree.mli14
-rw-r--r--lib/system.mli14
-rw-r--r--lib/tlm.mli14
-rw-r--r--lib/util.mli14
19 files changed, 133 insertions, 133 deletions
diff --git a/lib/bigint.mli b/lib/bigint.mli
index 348c6c5d9..82b43348e 100644
--- a/lib/bigint.mli
+++ b/lib/bigint.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
diff --git a/lib/dnet.mli b/lib/dnet.mli
index be33ecc6a..44cd76baf 100644
--- a/lib/dnet.mli
+++ b/lib/dnet.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 *)
+(************************************************************************)
(** Generic discrimination net implementation over recursive
types. This module implements a association data structure similar
diff --git a/lib/dyn.mli b/lib/dyn.mli
index 235dae3af..6a31c3bad 100644
--- a/lib/dyn.mli
+++ b/lib/dyn.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 *)
+(************************************************************************)
(** Dynamics. Use with extreme care. Not for kids. *)
diff --git a/lib/envars.mli b/lib/envars.mli
index 8e4ccb4d5..01abcbd4d 100644
--- a/lib/envars.mli
+++ b/lib/envars.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 *)
+(************************************************************************)
(** This file gathers environment variables needed by Coq to run (such
as coqlib) *)
diff --git a/lib/explore.mli b/lib/explore.mli
index 1f17f8a4c..3246eb19e 100644
--- a/lib/explore.mli
+++ b/lib/explore.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 *)
+(************************************************************************)
(** {6 Search strategies. } *)
diff --git a/lib/flags.mli b/lib/flags.mli
index 8576a7e5e..9ac1571ea 100644
--- a/lib/flags.mli
+++ b/lib/flags.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 *)
+(************************************************************************)
(** Global options of the system. *)
diff --git a/lib/gmap.mli b/lib/gmap.mli
index 45b04151e..626888d57 100644
--- a/lib/gmap.mli
+++ b/lib/gmap.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 *)
+(************************************************************************)
(** Maps using the generic comparison function of ocaml. Same interface as
the module [Map] from the ocaml standard library. *)
diff --git a/lib/gmapl.mli b/lib/gmapl.mli
index fdc42e3ad..add79d765 100644
--- a/lib/gmapl.mli
+++ b/lib/gmapl.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 *)
+(************************************************************************)
(** Maps from ['a] to lists of ['b]. *)
diff --git a/lib/gset.mli b/lib/gset.mli
index 265f8eb34..073942a0a 100644
--- a/lib/gset.mli
+++ b/lib/gset.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 *)
+(************************************************************************)
(** Sets using the generic comparison function of ocaml. Same interface as
the module [Set] from the ocaml standard library. *)
diff --git a/lib/hashcons.mli b/lib/hashcons.mli
index 2b3b7dfb0..6bdc04b37 100644
--- a/lib/hashcons.mli
+++ b/lib/hashcons.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 *)
+(************************************************************************)
(** Generic hash-consing. *)
diff --git a/lib/heap.mli b/lib/heap.mli
index fe34b250d..66e243ebb 100644
--- a/lib/heap.mli
+++ b/lib/heap.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 *)
+(************************************************************************)
(** Heaps *)
diff --git a/lib/option.mli b/lib/option.mli
index b37d905f5..c432f05d4 100644
--- a/lib/option.mli
+++ b/lib/option.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 *)
+(************************************************************************)
(** Module implementing basic combinators for OCaml option type.
It tries follow closely the style of OCaml standard library.
diff --git a/lib/pp.mli b/lib/pp.mli
index ca62f82d6..474285b67 100644
--- a/lib/pp.mli
+++ b/lib/pp.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_control
diff --git a/lib/pp_control.mli b/lib/pp_control.mli
index fe1ee6de3..21ea7a36d 100644
--- a/lib/pp_control.mli
+++ b/lib/pp_control.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 *)
+(************************************************************************)
(** Parameters of pretty-printing. *)
diff --git a/lib/profile.mli b/lib/profile.mli
index 1934b0482..5bcebfb0d 100644
--- a/lib/profile.mli
+++ b/lib/profile.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 *)
+(************************************************************************)
(** {6 This program is a small time and allocation profiler for Objective Caml } *)
diff --git a/lib/rtree.mli b/lib/rtree.mli
index 42723358d..b5559c62c 100644
--- a/lib/rtree.mli
+++ b/lib/rtree.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 *)
+(************************************************************************)
(** Type of regular tree with nodes labelled by values of type 'a
The implementation uses de Bruijn indices, so binding capture
diff --git a/lib/system.mli b/lib/system.mli
index 13fd09f5f..b1346653f 100644
--- a/lib/system.mli
+++ b/lib/system.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 *)
+(************************************************************************)
(** System utilities *)
diff --git a/lib/tlm.mli b/lib/tlm.mli
index e4c980696..73aa6132a 100644
--- a/lib/tlm.mli
+++ b/lib/tlm.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 *)
+(************************************************************************)
(** Tries. This module implements a data structure [('a,'b) t] mapping lists
of values of type ['a] to sets (as lists) of values of type ['b]. *)
diff --git a/lib/util.mli b/lib/util.mli
index 0976d742c..f8fbc1f68 100644
--- a/lib/util.mli
+++ b/lib/util.mli
@@ -1,10 +1,10 @@
-(**********************************************************************
- v * The Coq Proof Assistant / The Coq Development Team
- <O___,, * INRIA-Rocquencourt & LRI-CNRS-Orsay
- \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 Compat