aboutsummaryrefslogtreecommitdiffhomepage
path: root/kernel
diff options
context:
space:
mode:
authorGravatar filliatr <filliatr@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-03-15 13:38:59 +0000
committerGravatar filliatr <filliatr@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-03-15 13:38:59 +0000
commit187dc15532f0c6f380d7bcb07adc2180c29fedc2 (patch)
treed7bacf01519ca82b5745d2c493c7f7f1826106af /kernel
parent23741168b109daece8bb588b9c5fb4506e7726ce (diff)
entetes
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@1469 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'kernel')
-rw-r--r--kernel/closure.ml7
-rw-r--r--kernel/closure.mli7
-rw-r--r--kernel/cooking.ml7
-rw-r--r--kernel/cooking.mli7
-rw-r--r--kernel/declarations.ml7
-rw-r--r--kernel/declarations.mli7
-rw-r--r--kernel/environ.ml7
-rw-r--r--kernel/environ.mli7
-rw-r--r--kernel/esubst.ml7
-rw-r--r--kernel/esubst.mli7
-rw-r--r--kernel/evd.ml7
-rw-r--r--kernel/evd.mli7
-rw-r--r--kernel/indtypes.ml7
-rw-r--r--kernel/indtypes.mli7
-rw-r--r--kernel/inductive.ml7
-rw-r--r--kernel/inductive.mli7
-rw-r--r--kernel/instantiate.ml7
-rw-r--r--kernel/instantiate.mli7
-rw-r--r--kernel/names.ml7
-rw-r--r--kernel/names.mli7
-rw-r--r--kernel/reduction.ml7
-rw-r--r--kernel/reduction.mli7
-rw-r--r--kernel/safe_typing.ml7
-rw-r--r--kernel/safe_typing.mli7
-rw-r--r--kernel/sign.ml7
-rw-r--r--kernel/sign.mli7
-rw-r--r--kernel/term.ml7
-rw-r--r--kernel/term.mli7
-rw-r--r--kernel/type_errors.ml7
-rw-r--r--kernel/type_errors.mli7
-rw-r--r--kernel/typeops.ml7
-rw-r--r--kernel/typeops.mli7
-rw-r--r--kernel/univ.ml7
-rw-r--r--kernel/univ.mli7
34 files changed, 238 insertions, 0 deletions
diff --git a/kernel/closure.ml b/kernel/closure.ml
index ac8ed32eb..541cd7d59 100644
--- a/kernel/closure.ml
+++ b/kernel/closure.ml
@@ -1,3 +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 *)
+(***********************************************************************)
(* $Id$ *)
diff --git a/kernel/closure.mli b/kernel/closure.mli
index b4001f077..ef01b73bb 100644
--- a/kernel/closure.mli
+++ b/kernel/closure.mli
@@ -1,3 +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 *)
+(***********************************************************************)
(*i $Id$ i*)
diff --git a/kernel/cooking.ml b/kernel/cooking.ml
index f0be35882..2ad841d03 100644
--- a/kernel/cooking.ml
+++ b/kernel/cooking.ml
@@ -1,3 +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 *)
+(***********************************************************************)
(*i $Id$ i*)
diff --git a/kernel/cooking.mli b/kernel/cooking.mli
index 99327605b..f29503176 100644
--- a/kernel/cooking.mli
+++ b/kernel/cooking.mli
@@ -1,3 +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 *)
+(***********************************************************************)
(*i $Id$ i*)
diff --git a/kernel/declarations.ml b/kernel/declarations.ml
index 9de1866cc..da393b235 100644
--- a/kernel/declarations.ml
+++ b/kernel/declarations.ml
@@ -1,3 +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 *)
+(***********************************************************************)
(* $Id$ *)
diff --git a/kernel/declarations.mli b/kernel/declarations.mli
index 531a616ba..18566a0c3 100644
--- a/kernel/declarations.mli
+++ b/kernel/declarations.mli
@@ -1,3 +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 *)
+(***********************************************************************)
(*i $Id$ i*)
diff --git a/kernel/environ.ml b/kernel/environ.ml
index f88860935..d21d5b51c 100644
--- a/kernel/environ.ml
+++ b/kernel/environ.ml
@@ -1,3 +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 *)
+(***********************************************************************)
(* $Id$ *)
diff --git a/kernel/environ.mli b/kernel/environ.mli
index eba1e0979..953580b0f 100644
--- a/kernel/environ.mli
+++ b/kernel/environ.mli
@@ -1,3 +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 *)
+(***********************************************************************)
(*i $Id$ i*)
diff --git a/kernel/esubst.ml b/kernel/esubst.ml
index 0ab021e4c..7d24804cc 100644
--- a/kernel/esubst.ml
+++ b/kernel/esubst.ml
@@ -1,3 +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 *)
+(***********************************************************************)
(* $Id$ *)
diff --git a/kernel/esubst.mli b/kernel/esubst.mli
index ea5df0a28..284c2f32e 100644
--- a/kernel/esubst.mli
+++ b/kernel/esubst.mli
@@ -1,3 +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 *)
+(***********************************************************************)
(* $Id$ *)
diff --git a/kernel/evd.ml b/kernel/evd.ml
index 548f8b14a..9a4d5af6a 100644
--- a/kernel/evd.ml
+++ b/kernel/evd.ml
@@ -1,3 +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 *)
+(***********************************************************************)
(* $Id$ *)
diff --git a/kernel/evd.mli b/kernel/evd.mli
index 2353b6789..6c0e6a716 100644
--- a/kernel/evd.mli
+++ b/kernel/evd.mli
@@ -1,3 +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 *)
+(***********************************************************************)
(*i $Id$ i*)
diff --git a/kernel/indtypes.ml b/kernel/indtypes.ml
index 228e2bafa..e67aff002 100644
--- a/kernel/indtypes.ml
+++ b/kernel/indtypes.ml
@@ -1,3 +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 *)
+(***********************************************************************)
(* $Id$ *)
diff --git a/kernel/indtypes.mli b/kernel/indtypes.mli
index d0e3a4cb0..f5a6ca236 100644
--- a/kernel/indtypes.mli
+++ b/kernel/indtypes.mli
@@ -1,3 +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 *)
+(***********************************************************************)
(*i $Id$ i*)
diff --git a/kernel/inductive.ml b/kernel/inductive.ml
index f03b1ba14..9a8ed21d8 100644
--- a/kernel/inductive.ml
+++ b/kernel/inductive.ml
@@ -1,3 +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 *)
+(***********************************************************************)
(* $Id$ *)
diff --git a/kernel/inductive.mli b/kernel/inductive.mli
index e1ee0a56f..00c0dfbdb 100644
--- a/kernel/inductive.mli
+++ b/kernel/inductive.mli
@@ -1,3 +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 *)
+(***********************************************************************)
(*i $Id$ i*)
diff --git a/kernel/instantiate.ml b/kernel/instantiate.ml
index c73fbd220..a92de9e60 100644
--- a/kernel/instantiate.ml
+++ b/kernel/instantiate.ml
@@ -1,3 +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 *)
+(***********************************************************************)
(* $Id$ *)
diff --git a/kernel/instantiate.mli b/kernel/instantiate.mli
index 9b083293a..14a4746ee 100644
--- a/kernel/instantiate.mli
+++ b/kernel/instantiate.mli
@@ -1,3 +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 *)
+(***********************************************************************)
(*i $Id$ i*)
diff --git a/kernel/names.ml b/kernel/names.ml
index 035a5d505..b4b6c4302 100644
--- a/kernel/names.ml
+++ b/kernel/names.ml
@@ -1,3 +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 *)
+(***********************************************************************)
(* $Id$ *)
diff --git a/kernel/names.mli b/kernel/names.mli
index 98e39fae9..6b817e683 100644
--- a/kernel/names.mli
+++ b/kernel/names.mli
@@ -1,3 +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 *)
+(***********************************************************************)
(*i $Id$ i*)
diff --git a/kernel/reduction.ml b/kernel/reduction.ml
index 7c244c280..a92fe89ee 100644
--- a/kernel/reduction.ml
+++ b/kernel/reduction.ml
@@ -1,3 +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 *)
+(***********************************************************************)
(* $Id$ *)
diff --git a/kernel/reduction.mli b/kernel/reduction.mli
index 794c49354..20435a1fc 100644
--- a/kernel/reduction.mli
+++ b/kernel/reduction.mli
@@ -1,3 +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 *)
+(***********************************************************************)
(*i $Id$ i*)
diff --git a/kernel/safe_typing.ml b/kernel/safe_typing.ml
index cb85a9868..ec3b75523 100644
--- a/kernel/safe_typing.ml
+++ b/kernel/safe_typing.ml
@@ -1,3 +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 *)
+(***********************************************************************)
(* $Id$ *)
diff --git a/kernel/safe_typing.mli b/kernel/safe_typing.mli
index 474da34b8..90703ae96 100644
--- a/kernel/safe_typing.mli
+++ b/kernel/safe_typing.mli
@@ -1,3 +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 *)
+(***********************************************************************)
(*i $Id$ i*)
diff --git a/kernel/sign.ml b/kernel/sign.ml
index fc3e15f5e..dff7e1218 100644
--- a/kernel/sign.ml
+++ b/kernel/sign.ml
@@ -1,3 +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 *)
+(***********************************************************************)
(* $Id$ *)
diff --git a/kernel/sign.mli b/kernel/sign.mli
index ede431eb4..6180906cb 100644
--- a/kernel/sign.mli
+++ b/kernel/sign.mli
@@ -1,3 +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 *)
+(***********************************************************************)
(*i $Id$ i*)
diff --git a/kernel/term.ml b/kernel/term.ml
index 66f706895..99e41ae56 100644
--- a/kernel/term.ml
+++ b/kernel/term.ml
@@ -1,3 +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 *)
+(***********************************************************************)
(* $Id$ *)
diff --git a/kernel/term.mli b/kernel/term.mli
index 87a6c06f6..b160594f1 100644
--- a/kernel/term.mli
+++ b/kernel/term.mli
@@ -1,3 +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 *)
+(***********************************************************************)
(*i $Id$ i*)
diff --git a/kernel/type_errors.ml b/kernel/type_errors.ml
index bf0a99ee3..387b7a930 100644
--- a/kernel/type_errors.ml
+++ b/kernel/type_errors.ml
@@ -1,3 +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 *)
+(***********************************************************************)
(* $Id$ *)
diff --git a/kernel/type_errors.mli b/kernel/type_errors.mli
index c45fac721..e022be01d 100644
--- a/kernel/type_errors.mli
+++ b/kernel/type_errors.mli
@@ -1,3 +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 *)
+(***********************************************************************)
(*i $Id$ i*)
diff --git a/kernel/typeops.ml b/kernel/typeops.ml
index 694d9ae77..17f30408d 100644
--- a/kernel/typeops.ml
+++ b/kernel/typeops.ml
@@ -1,3 +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 *)
+(***********************************************************************)
(* $Id$ *)
diff --git a/kernel/typeops.mli b/kernel/typeops.mli
index f06e65653..b2db98373 100644
--- a/kernel/typeops.mli
+++ b/kernel/typeops.mli
@@ -1,3 +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 *)
+(***********************************************************************)
(*i $Id$ i*)
diff --git a/kernel/univ.ml b/kernel/univ.ml
index 4ea2ded00..fc5e4ff23 100644
--- a/kernel/univ.ml
+++ b/kernel/univ.ml
@@ -1,3 +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 *)
+(***********************************************************************)
(* $Id$ *)
diff --git a/kernel/univ.mli b/kernel/univ.mli
index 2460ff15e..3aedf921e 100644
--- a/kernel/univ.mli
+++ b/kernel/univ.mli
@@ -1,3 +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 *)
+(***********************************************************************)
(*i $Id$ i*)