diff options
175 files changed, 1250 insertions, 1221 deletions
diff --git a/dev/tools/change-header b/dev/tools/change-header new file mode 100755 index 000000000..8b3560e89 --- /dev/null +++ b/dev/tools/change-header @@ -0,0 +1,32 @@ +#!/bin/sh + +#This script changes the header of .ml* files + +if [ ! $# = 2 ]; then + echo Usage: change-header old-header-file new-header-file + exit 1 +fi + +oldheader=$1 +newheader=$2 + +if [ ! -f $oldheader ]; then echo Cannot read file $oldheader; exit 1; fi +if [ ! -f $newheader ]; then echo Cannot read file $newheader; exit 1; fi + +n=`wc -l $oldheader | sed -e "s/ *\([0-9]*\).*/\1/g"` +nsucc=`expr $n + 1` + +filter="-name \*.mli -o -name \*.ml -o -name \*.ml4 -o -name \*.mll -o -name \*.mly" + +for i in `find . $filter`; do + head -n +$n $i > $i.head.tmp$$ + if diff -a -q $oldheader $i.head.tmp$$ > /dev/null; then + rm $i.head.tmp$$ + echo "$i: header changed" + cat dev/header > $i.tmp$$ + tail -n +$nsucc $i >> $i.tmp$$ + mv $i.tmp$$ $i + else + echo "$i: old header not found, file untouched" + fi +done 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 diff --git a/kernel/closure.mli b/kernel/closure.mli index 9a8ced44e..7becd7c63 100644 --- a/kernel/closure.mli +++ b/kernel/closure.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/kernel/conv_oracle.mli b/kernel/conv_oracle.mli index 0e8201694..1c953d28f 100644 --- a/kernel/conv_oracle.mli +++ b/kernel/conv_oracle.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 diff --git a/kernel/cooking.mli b/kernel/cooking.mli index 42991d507..2ca7b17d8 100644 --- a/kernel/cooking.mli +++ b/kernel/cooking.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/kernel/declarations.mli b/kernel/declarations.mli index 36af9dc48..de8b081b7 100644 --- a/kernel/declarations.mli +++ b/kernel/declarations.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 Univ diff --git a/kernel/entries.mli b/kernel/entries.mli index 78316dd9b..001bc72fe 100644 --- a/kernel/entries.mli +++ b/kernel/entries.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 Univ diff --git a/kernel/environ.mli b/kernel/environ.mli index 8c31742f3..e1d09e1dc 100644 --- a/kernel/environ.mli +++ b/kernel/environ.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/kernel/esubst.mli b/kernel/esubst.mli index dd7096c4b..73eba7ecd 100644 --- a/kernel/esubst.mli +++ b/kernel/esubst.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 *) +(************************************************************************) (** Explicit substitutions *) diff --git a/kernel/indtypes.mli b/kernel/indtypes.mli index 40d6912c4..306c407c7 100644 --- a/kernel/indtypes.mli +++ b/kernel/indtypes.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 Univ diff --git a/kernel/inductive.mli b/kernel/inductive.mli index 42a2da41b..91afda7c3 100644 --- a/kernel/inductive.mli +++ b/kernel/inductive.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 Univ diff --git a/kernel/mod_subst.mli b/kernel/mod_subst.mli index 2514e409c..922ffaf4a 100644 --- a/kernel/mod_subst.mli +++ b/kernel/mod_subst.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 [Mod_subst] } *) diff --git a/kernel/mod_typing.mli b/kernel/mod_typing.mli index 10619820e..3027a6293 100644 --- a/kernel/mod_typing.mli +++ b/kernel/mod_typing.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/kernel/modops.mli b/kernel/modops.mli index 3ab2961d2..cfa5f9cd9 100644 --- a/kernel/modops.mli +++ b/kernel/modops.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/kernel/names.mli b/kernel/names.mli index 74cebd22a..b441bf00a 100644 --- a/kernel/names.mli +++ b/kernel/names.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 Identifiers } *) diff --git a/kernel/pre_env.mli b/kernel/pre_env.mli index 9078558a9..8c6e69fac 100644 --- a/kernel/pre_env.mli +++ b/kernel/pre_env.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/kernel/reduction.mli b/kernel/reduction.mli index ced0fd341..dc29d1454 100644 --- a/kernel/reduction.mli +++ b/kernel/reduction.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 Term open Environ diff --git a/kernel/retroknowledge.mli b/kernel/retroknowledge.mli index 0634a99aa..3349a81bc 100644 --- a/kernel/retroknowledge.mli +++ b/kernel/retroknowledge.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/kernel/safe_typing.mli b/kernel/safe_typing.mli index 3e1051088..a80423272 100644 --- a/kernel/safe_typing.mli +++ b/kernel/safe_typing.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/kernel/sign.mli b/kernel/sign.mli index ddb88287e..4953ff835 100644 --- a/kernel/sign.mli +++ b/kernel/sign.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/kernel/subtyping.mli b/kernel/subtyping.mli index 061a6eb0b..89d532cfd 100644 --- a/kernel/subtyping.mli +++ b/kernel/subtyping.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 Univ open Declarations diff --git a/kernel/term.mli b/kernel/term.mli index 5efd95696..12570a434 100644 --- a/kernel/term.mli +++ b/kernel/term.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 diff --git a/kernel/term_typing.mli b/kernel/term_typing.mli index dbf479a0c..16adbfb3d 100644 --- a/kernel/term_typing.mli +++ b/kernel/term_typing.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/kernel/type_errors.mli b/kernel/type_errors.mli index 3a6ad4bb1..5b119159a 100644 --- a/kernel/type_errors.mli +++ b/kernel/type_errors.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/kernel/typeops.mli b/kernel/typeops.mli index e2df7e983..a6a04aa85 100644 --- a/kernel/typeops.mli +++ b/kernel/typeops.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 Univ diff --git a/kernel/univ.mli b/kernel/univ.mli index 1634009b3..3965959d0 100644 --- a/kernel/univ.mli +++ b/kernel/univ.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 *) +(************************************************************************) (** Universes. *) diff --git a/kernel/vconv.mli b/kernel/vconv.mli index 6776821ed..405ef7a33 100644 --- a/kernel/vconv.mli +++ b/kernel/vconv.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/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 diff --git a/library/decl_kinds.mli b/library/decl_kinds.mli index 2c04d0fdd..bdf01bfc0 100644 --- a/library/decl_kinds.mli +++ b/library/decl_kinds.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 Libnames diff --git a/library/declare.mli b/library/declare.mli index db9e1aa6d..3ff91cc5e 100644 --- a/library/declare.mli +++ b/library/declare.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/library/declaremods.mli b/library/declaremods.mli index b7126147e..de12c036c 100644 --- a/library/declaremods.mli +++ b/library/declaremods.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/library/decls.mli b/library/decls.mli index 34a96cd8b..641038d55 100644 --- a/library/decls.mli +++ b/library/decls.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 Sign diff --git a/library/dischargedhypsmap.mli b/library/dischargedhypsmap.mli index 98e3d93d5..8284e68a2 100644 --- a/library/dischargedhypsmap.mli +++ b/library/dischargedhypsmap.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 Libnames open Term diff --git a/library/global.mli b/library/global.mli index d29aca5d3..97024a40b 100644 --- a/library/global.mli +++ b/library/global.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 Univ diff --git a/library/goptions.mli b/library/goptions.mli index c63845ae0..72a16c026 100644 --- a/library/goptions.mli +++ b/library/goptions.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 module manages customization parameters at the vernacular level *) diff --git a/library/heads.mli b/library/heads.mli index 5a0df8423..4598a21ea 100644 --- a/library/heads.mli +++ b/library/heads.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/library/impargs.mli b/library/impargs.mli index 2eab1af66..74c33dc04 100644 --- a/library/impargs.mli +++ b/library/impargs.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/library/lib.mli b/library/lib.mli index 5fb65a41f..9a0a0ddaf 100644 --- a/library/lib.mli +++ b/library/lib.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 *) +(************************************************************************) (** Lib: record of operations, backtrack, low-level sections *) diff --git a/library/libnames.mli b/library/libnames.mli index 4e9ddcb56..d4f70fde0 100644 --- a/library/libnames.mli +++ b/library/libnames.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 diff --git a/library/libobject.mli b/library/libobject.mli index 87bbbe89d..471416df0 100644 --- a/library/libobject.mli +++ b/library/libobject.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/library/library.mli b/library/library.mli index 87e376ab9..7fc613aa0 100644 --- a/library/library.mli +++ b/library/library.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/library/nameops.mli b/library/nameops.mli index 121f0ce77..13e01306b 100644 --- a/library/nameops.mli +++ b/library/nameops.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 diff --git a/library/nametab.mli b/library/nametab.mli index 2f81ff50e..9019e27ab 100755..100644 --- a/library/nametab.mli +++ b/library/nametab.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/library/states.mli b/library/states.mli index 9b5872bde..bacc9fb76 100644 --- a/library/states.mli +++ b/library/states.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 States of the system} *) diff --git a/library/summary.mli b/library/summary.mli index 0f6aaddaf..0ef3b6f30 100644 --- a/library/summary.mli +++ b/library/summary.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 module registers the declaration of global tables, which will be kept in synchronization during the various backtracks of the system. *) diff --git a/parsing/egrammar.mli b/parsing/egrammar.mli index a0004ce38..56e6b1d61 100644 --- a/parsing/egrammar.mli +++ b/parsing/egrammar.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 Compat open Util diff --git a/parsing/extend.mli b/parsing/extend.mli index 597ff69a5..a05952294 100644 --- a/parsing/extend.mli +++ b/parsing/extend.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 Compat diff --git a/parsing/extrawit.mli b/parsing/extrawit.mli index b330a8e64..83b8a95ff 100644 --- a/parsing/extrawit.mli +++ b/parsing/extrawit.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 Genarg diff --git a/parsing/g_intsyntax.mli b/parsing/g_intsyntax.mli index 40e16b83c..5db25305e 100644 --- a/parsing/g_intsyntax.mli +++ b/parsing/g_intsyntax.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 *) +(************************************************************************) (*i $$ i*) diff --git a/parsing/g_natsyntax.mli b/parsing/g_natsyntax.mli index 3751f603b..8f9b3f904 100644 --- a/parsing/g_natsyntax.mli +++ b/parsing/g_natsyntax.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 *) +(************************************************************************) (** Nice syntax for naturals. *) diff --git a/parsing/g_zsyntax.mli b/parsing/g_zsyntax.mli index 29dd60f35..6e81af28c 100644 --- a/parsing/g_zsyntax.mli +++ b/parsing/g_zsyntax.mli @@ -1,9 +1,9 @@ -(*********************************************************************** - 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 *) +(************************************************************************) (** Nice syntax for integers. *) diff --git a/parsing/lexer.mli b/parsing/lexer.mli index a8ae46fec..0e8be6895 100644 --- a/parsing/lexer.mli +++ b/parsing/lexer.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 diff --git a/parsing/pcoq.mli b/parsing/pcoq.mli index 31adbd6c0..1436b0e18 100644 --- a/parsing/pcoq.mli +++ b/parsing/pcoq.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/parsing/ppconstr.mli b/parsing/ppconstr.mli index afa744a50..59c1f3af7 100644 --- a/parsing/ppconstr.mli +++ b/parsing/ppconstr.mli @@ -1,11 +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 Environ diff --git a/parsing/pptactic.mli b/parsing/pptactic.mli index 34a7089fe..60e3648ab 100644 --- a/parsing/pptactic.mli +++ b/parsing/pptactic.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 Genarg diff --git a/parsing/ppvernac.mli b/parsing/ppvernac.mli index 98511f3e5..80109af1e 100644 --- a/parsing/ppvernac.mli +++ b/parsing/ppvernac.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 Genarg diff --git a/parsing/prettyp.mli b/parsing/prettyp.mli index 913ab8b43..0a4c14944 100644 --- a/parsing/prettyp.mli +++ b/parsing/prettyp.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 diff --git a/parsing/printer.mli b/parsing/printer.mli index 241650b7d..c41dabf7d 100644 --- a/parsing/printer.mli +++ b/parsing/printer.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/parsing/printmod.mli b/parsing/printmod.mli index b7926543d..d99b44728 100644 --- a/parsing/printmod.mli +++ b/parsing/printmod.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/parsing/q_util.mli b/parsing/q_util.mli index c19a0ecf5..166b00521 100644 --- a/parsing/q_util.mli +++ b/parsing/q_util.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 Compat diff --git a/parsing/tactic_printer.mli b/parsing/tactic_printer.mli index 129f0e671..60a47b75a 100644 --- a/parsing/tactic_printer.mli +++ b/parsing/tactic_printer.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 Sign diff --git a/parsing/tok.ml b/parsing/tok.ml index 870f2d5e7..55cbdecb9 100644 --- a/parsing/tok.ml +++ b/parsing/tok.ml @@ -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 *) +(************************************************************************) (** The type of token for the Coq lexer and parser *) diff --git a/parsing/tok.mli b/parsing/tok.mli index 0e2730b17..3764ef539 100644 --- a/parsing/tok.mli +++ b/parsing/tok.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 *) +(************************************************************************) (** The type of token for the Coq lexer and parser *) diff --git a/pretyping/cases.mli b/pretyping/cases.mli index cc064bc4d..1d8df523f 100644 --- a/pretyping/cases.mli +++ b/pretyping/cases.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/pretyping/cbv.mli b/pretyping/cbv.mli index 50b4fda4a..5c0ff6027 100644 --- a/pretyping/cbv.mli +++ b/pretyping/cbv.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/pretyping/classops.mli b/pretyping/classops.mli index 6184ed7a1..ba6eb4ca6 100644 --- a/pretyping/classops.mli +++ b/pretyping/classops.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/pretyping/coercion.mli b/pretyping/coercion.mli index a5ed740f9..7da8851f6 100644 --- a/pretyping/coercion.mli +++ b/pretyping/coercion.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 Evd diff --git a/pretyping/detyping.mli b/pretyping/detyping.mli index 47a7beb53..ebca020ab 100644 --- a/pretyping/detyping.mli +++ b/pretyping/detyping.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/pretyping/evarconv.mli b/pretyping/evarconv.mli index 1ddf97c86..578318a83 100644 --- a/pretyping/evarconv.mli +++ b/pretyping/evarconv.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 Term open Sign diff --git a/pretyping/evarutil.mli b/pretyping/evarutil.mli index e21516681..1d11097d3 100644 --- a/pretyping/evarutil.mli +++ b/pretyping/evarutil.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/pretyping/evd.mli b/pretyping/evd.mli index 87e703463..24d865beb 100644 --- a/pretyping/evd.mli +++ b/pretyping/evd.mli @@ -1,11 +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/pretyping/indrec.mli b/pretyping/indrec.mli index 7f19c5d37..511ec9c51 100644 --- a/pretyping/indrec.mli +++ b/pretyping/indrec.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/pretyping/inductiveops.mli b/pretyping/inductiveops.mli index 98a22fabd..7c5642d1d 100644 --- a/pretyping/inductiveops.mli +++ b/pretyping/inductiveops.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/pretyping/matching.mli b/pretyping/matching.mli index eb9c8fc8c..86657d287 100644 --- a/pretyping/matching.mli +++ b/pretyping/matching.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 module implements pattern-matching on terms *) diff --git a/pretyping/namegen.mli b/pretyping/namegen.mli index 889f8ec8c..5560cddf7 100644 --- a/pretyping/namegen.mli +++ b/pretyping/namegen.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/pretyping/pattern.mli b/pretyping/pattern.mli index 3b61c1e43..5685f3d2c 100644 --- a/pretyping/pattern.mli +++ b/pretyping/pattern.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 module defines the type of pattern used for pattern-matching terms in tatics *) diff --git a/pretyping/pretype_errors.mli b/pretyping/pretype_errors.mli index f55e70bef..0bdbb1c65 100644 --- a/pretyping/pretype_errors.mli +++ b/pretyping/pretype_errors.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 diff --git a/pretyping/pretyping.mli b/pretyping/pretyping.mli index 00eb613ab..d6996dd3b 100644 --- a/pretyping/pretyping.mli +++ b/pretyping/pretyping.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 implements type inference. It maps [rawconstr] (i.e. untyped terms whose names are located) to [constr]. In diff --git a/pretyping/rawterm.mli b/pretyping/rawterm.mli index 0c8f15472..d7f8311c7 100644 --- a/pretyping/rawterm.mli +++ b/pretyping/rawterm.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 *) +(************************************************************************) (**Untyped intermediate terms, after constr_expr and before constr diff --git a/pretyping/recordops.mli b/pretyping/recordops.mli index 5651b7687..6ad5fbc64 100755..100644 --- a/pretyping/recordops.mli +++ b/pretyping/recordops.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 Nametab diff --git a/pretyping/reductionops.mli b/pretyping/reductionops.mli index 4518c693d..40c0e2813 100644 --- a/pretyping/reductionops.mli +++ b/pretyping/reductionops.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/pretyping/retyping.mli b/pretyping/retyping.mli index 5b445ff9c..2733b1473 100644 --- a/pretyping/retyping.mli +++ b/pretyping/retyping.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/pretyping/tacred.mli b/pretyping/tacred.mli index fdceadfbb..4793027fb 100644 --- a/pretyping/tacred.mli +++ b/pretyping/tacred.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/pretyping/term_dnet.mli b/pretyping/term_dnet.mli index 3db55b162..242fc8cd7 100644 --- a/pretyping/term_dnet.mli +++ b/pretyping/term_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 *) +(************************************************************************) open Term open Sign diff --git a/pretyping/termops.mli b/pretyping/termops.mli index 050084bb1..fc227b5fb 100644 --- a/pretyping/termops.mli +++ b/pretyping/termops.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/pretyping/typeclasses.mli b/pretyping/typeclasses.mli index dc1c5f556..ebdfe25c4 100644 --- a/pretyping/typeclasses.mli +++ b/pretyping/typeclasses.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/pretyping/typeclasses_errors.mli b/pretyping/typeclasses_errors.mli index 43b349515..8f21510b0 100644 --- a/pretyping/typeclasses_errors.mli +++ b/pretyping/typeclasses_errors.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/pretyping/typing.mli b/pretyping/typing.mli index 90f823b8e..9bfc26057 100644 --- a/pretyping/typing.mli +++ b/pretyping/typing.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 Term open Environ diff --git a/pretyping/unification.mli b/pretyping/unification.mli index 8829d8989..8cd7003ed 100644 --- a/pretyping/unification.mli +++ b/pretyping/unification.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 Term open Environ diff --git a/pretyping/vnorm.mli b/pretyping/vnorm.mli index da9e7cf1e..2820b1b4f 100644 --- a/pretyping/vnorm.mli +++ b/pretyping/vnorm.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/proofs/clenv.mli b/proofs/clenv.mli index 9a93adc44..cd1bbde53 100644 --- a/proofs/clenv.mli +++ b/proofs/clenv.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/proofs/clenvtac.mli b/proofs/clenvtac.mli index 760a79d4c..d3cf2a436 100644 --- a/proofs/clenvtac.mli +++ b/proofs/clenvtac.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/proofs/evar_refiner.mli b/proofs/evar_refiner.mli index a8debc6fd..559152e8b 100644 --- a/proofs/evar_refiner.mli +++ b/proofs/evar_refiner.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/proofs/logic.mli b/proofs/logic.mli index 39f69ad12..6ad50f4b4 100644 --- a/proofs/logic.mli +++ b/proofs/logic.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/proofs/pfedit.mli b/proofs/pfedit.mli index f95721a7a..bc80e7eeb 100644 --- a/proofs/pfedit.mli +++ b/proofs/pfedit.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/proofs/proof_type.mli b/proofs/proof_type.mli index 73be0c2b7..0a3015844 100644 --- a/proofs/proof_type.mli +++ b/proofs/proof_type.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 Environ open Evd diff --git a/proofs/redexpr.mli b/proofs/redexpr.mli index 581ee1dc9..11aa0af36 100644 --- a/proofs/redexpr.mli +++ b/proofs/redexpr.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/proofs/refiner.mli b/proofs/refiner.mli index be4dbd9a5..74f9dc9ec 100644 --- a/proofs/refiner.mli +++ b/proofs/refiner.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 Term open Sign diff --git a/proofs/tacmach.mli b/proofs/tacmach.mli index 9e0ca2a3d..90de6166d 100644 --- a/proofs/tacmach.mli +++ b/proofs/tacmach.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/proofs/tactic_debug.mli b/proofs/tactic_debug.mli index ac3bf493a..557e658ac 100644 --- a/proofs/tactic_debug.mli +++ b/proofs/tactic_debug.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 Environ open Pattern diff --git a/tactics/auto.mli b/tactics/auto.mli index 684478d96..d42e541c0 100644 --- a/tactics/auto.mli +++ b/tactics/auto.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/tactics/autorewrite.mli b/tactics/autorewrite.mli index bda1fc65f..5ab803872 100644 --- a/tactics/autorewrite.mli +++ b/tactics/autorewrite.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 Term open Tacexpr diff --git a/tactics/btermdn.mli b/tactics/btermdn.mli index a4ace7637..928acdac1 100644 --- a/tactics/btermdn.mli +++ b/tactics/btermdn.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 Term open Pattern diff --git a/tactics/contradiction.mli b/tactics/contradiction.mli index b74a23271..d77fbde3a 100644 --- a/tactics/contradiction.mli +++ b/tactics/contradiction.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/tactics/dhyp.mli b/tactics/dhyp.mli index c35b4d759..982dc7ec9 100644 --- a/tactics/dhyp.mli +++ b/tactics/dhyp.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 Tacmach diff --git a/tactics/eauto.mli b/tactics/eauto.mli index b51cb9d4b..74bbb8b45 100644 --- a/tactics/eauto.mli +++ b/tactics/eauto.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 Term open Proof_type diff --git a/tactics/elim.mli b/tactics/elim.mli index 2351947e0..20ad0d579 100644 --- a/tactics/elim.mli +++ b/tactics/elim.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/tactics/elimschemes.mli b/tactics/elimschemes.mli index d58878838..e3944a266 100644 --- a/tactics/elimschemes.mli +++ b/tactics/elimschemes.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 Ind_tables diff --git a/tactics/eqschemes.mli b/tactics/eqschemes.mli index 3d0ea4790..cbd146659 100644 --- a/tactics/eqschemes.mli +++ b/tactics/eqschemes.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 builds schemes relative to equality inductive types *) diff --git a/tactics/evar_tactics.mli b/tactics/evar_tactics.mli index ffce59547..29f72d1af 100644 --- a/tactics/evar_tactics.mli +++ b/tactics/evar_tactics.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 Tacmach open Names diff --git a/tactics/extraargs.mli b/tactics/extraargs.mli index 2c750be36..c0310b448 100644 --- a/tactics/extraargs.mli +++ b/tactics/extraargs.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 Tacexpr open Term diff --git a/tactics/extratactics.mli b/tactics/extratactics.mli index f2f13fe11..4d0e69fcb 100644 --- a/tactics/extratactics.mli +++ b/tactics/extratactics.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 Proof_type diff --git a/tactics/hiddentac.mli b/tactics/hiddentac.mli index 120d42abf..afc1f63eb 100644 --- a/tactics/hiddentac.mli +++ b/tactics/hiddentac.mli @@ -1,11 +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 Util diff --git a/tactics/hipattern.mli b/tactics/hipattern.mli index c44eb6fdd..fba2b6650 100644 --- a/tactics/hipattern.mli +++ b/tactics/hipattern.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/tactics/inv.mli b/tactics/inv.mli index b038e4f0e..b2d416a6f 100644 --- a/tactics/inv.mli +++ b/tactics/inv.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/tactics/nbtermdn.mli b/tactics/nbtermdn.mli index 1dae56052..f06e4fc7a 100644 --- a/tactics/nbtermdn.mli +++ b/tactics/nbtermdn.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 Term open Pattern diff --git a/tactics/refine.mli b/tactics/refine.mli index ef369a857..09fea6d5b 100644 --- a/tactics/refine.mli +++ b/tactics/refine.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 Tacmach diff --git a/tactics/tacinterp.mli b/tactics/tacinterp.mli index 9909b6d68..a591c4331 100644 --- a/tactics/tacinterp.mli +++ b/tactics/tacinterp.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 diff --git a/tactics/tacticals.mli b/tactics/tacticals.mli index e67e11227..bfcb4e489 100644 --- a/tactics/tacticals.mli +++ b/tactics/tacticals.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 diff --git a/tactics/tactics.mli b/tactics/tactics.mli index 8a413e137..fa052ae6a 100644 --- a/tactics/tactics.mli +++ b/tactics/tactics.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/tactics/termdn.mli b/tactics/termdn.mli index 1453fdadb..244984a91 100644 --- a/tactics/termdn.mli +++ b/tactics/termdn.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 Term open Pattern diff --git a/toplevel/auto_ind_decl.mli b/toplevel/auto_ind_decl.mli index 901ddb721..589173a07 100644 --- a/toplevel/auto_ind_decl.mli +++ b/toplevel/auto_ind_decl.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 Term open Names diff --git a/toplevel/autoinstance.mli b/toplevel/autoinstance.mli index 4f1787e14..fa5360eeb 100644 --- a/toplevel/autoinstance.mli +++ b/toplevel/autoinstance.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 Term open Libnames diff --git a/toplevel/cerrors.mli b/toplevel/cerrors.mli index e95c07c61..c5c30eac1 100644 --- a/toplevel/cerrors.mli +++ b/toplevel/cerrors.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 diff --git a/toplevel/class.mli b/toplevel/class.mli index 51fb8b26e..7a0bf196b 100644 --- a/toplevel/class.mli +++ b/toplevel/class.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/toplevel/classes.mli b/toplevel/classes.mli index cae779b08..9a480075b 100644 --- a/toplevel/classes.mli +++ b/toplevel/classes.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/toplevel/command.mli b/toplevel/command.mli index 3a6bb18c1..b056afa58 100644 --- a/toplevel/command.mli +++ b/toplevel/command.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/toplevel/coqinit.mli b/toplevel/coqinit.mli index f209fd738..a306057b8 100644 --- a/toplevel/coqinit.mli +++ b/toplevel/coqinit.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 *) +(************************************************************************) (** Initialization. *) diff --git a/toplevel/coqtop.mli b/toplevel/coqtop.mli index 104e964c2..269997301 100644 --- a/toplevel/coqtop.mli +++ b/toplevel/coqtop.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 *) +(************************************************************************) (** The Coq main module. The following function [start] will parse the command line, print the banner, initialize the load path, load the input diff --git a/toplevel/discharge.mli b/toplevel/discharge.mli index 03f831c23..c856c1c17 100644 --- a/toplevel/discharge.mli +++ b/toplevel/discharge.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 Sign open Cooking diff --git a/toplevel/himsg.mli b/toplevel/himsg.mli index 464c8f89c..b2f86d6e9 100644 --- a/toplevel/himsg.mli +++ b/toplevel/himsg.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/toplevel/ind_tables.mli b/toplevel/ind_tables.mli index 2abd15ce3..0d3a250c9 100644 --- a/toplevel/ind_tables.mli +++ b/toplevel/ind_tables.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 Term open Names diff --git a/toplevel/indschemes.mli b/toplevel/indschemes.mli index 291b66776..ec055933d 100644 --- a/toplevel/indschemes.mli +++ b/toplevel/indschemes.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/toplevel/lemmas.mli b/toplevel/lemmas.mli index 40a1d802c..54b69f941 100644 --- a/toplevel/lemmas.mli +++ b/toplevel/lemmas.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.fix_expr - ***********************************************************************) +(************************************************************************) +(* 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/toplevel/libtypes.mli b/toplevel/libtypes.mli index 5d0fcfee6..cb495a30a 100644 --- a/toplevel/libtypes.mli +++ b/toplevel/libtypes.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 Term diff --git a/toplevel/metasyntax.mli b/toplevel/metasyntax.mli index f558fc4d1..216d03381 100644 --- a/toplevel/metasyntax.mli +++ b/toplevel/metasyntax.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/toplevel/mltop.mli b/toplevel/mltop.mli index 9da357581..363428b3b 100644 --- a/toplevel/mltop.mli +++ b/toplevel/mltop.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 *) +(************************************************************************) (** If there is a toplevel under Coq, it is described by the following record. *) diff --git a/toplevel/record.mli b/toplevel/record.mli index 2090cf1e5..b4c5a3375 100644 --- a/toplevel/record.mli +++ b/toplevel/record.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/toplevel/search.mli b/toplevel/search.mli index 28096eb5e..74f92e323 100644 --- a/toplevel/search.mli +++ b/toplevel/search.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/toplevel/toplevel.mli b/toplevel/toplevel.mli index 8980ef92b..350a9826b 100644 --- a/toplevel/toplevel.mli +++ b/toplevel/toplevel.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 Pcoq diff --git a/toplevel/usage.mli b/toplevel/usage.mli index 23e807c16..a667f3052 100644 --- a/toplevel/usage.mli +++ b/toplevel/usage.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 Prints the version number on the standard output and exits (with 0). } *) diff --git a/toplevel/vernac.mli b/toplevel/vernac.mli index 01852f130..5ce1d672e 100644 --- a/toplevel/vernac.mli +++ b/toplevel/vernac.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 *) +(************************************************************************) (** Parsing of vernacular. *) diff --git a/toplevel/vernacentries.mli b/toplevel/vernacentries.mli index b70eb61fb..fce6ef1f9 100644 --- a/toplevel/vernacentries.mli +++ b/toplevel/vernacentries.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/toplevel/vernacinterp.mli b/toplevel/vernacinterp.mli index 0a58b17b5..f8959fa3b 100644 --- a/toplevel/vernacinterp.mli +++ b/toplevel/vernacinterp.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 Tacexpr diff --git a/toplevel/whelp.mli b/toplevel/whelp.mli index 72245021d..105688bdf 100644 --- a/toplevel/whelp.mli +++ b/toplevel/whelp.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 *) +(************************************************************************) (** Coq interface to the Whelp query engine developed at the University of Bologna *) |