aboutsummaryrefslogtreecommitdiff
diff options
context:
space:
mode:
authorThéo Zimmermann2020-03-18 11:45:56 +0100
committerThéo Zimmermann2020-03-18 11:45:56 +0100
commite92ae479c6f370a865deff196df60efffd1c9125 (patch)
tree6a5d1cad8f139cf3a6cb5f15e5d0a038f4eee901
parent693c0fb3ad7344aadc840ab7124782e64997b739 (diff)
Remove dates in headers.
Cf. discussion at #11559 and decision of Coq Call 2020-02-26.
-rw-r--r--dev/header.c4
-rw-r--r--dev/header.ml4
-rw-r--r--dev/header.py4
3 files changed, 6 insertions, 6 deletions
diff --git a/dev/header.c b/dev/header.c
index 6201cb3b73..f31efcba47 100644
--- a/dev/header.c
+++ b/dev/header.c
@@ -1,7 +1,7 @@
/************************************************************************/
/* * The Coq Proof Assistant / The Coq Development Team */
-/* v * INRIA, CNRS and contributors - Copyright 1999-2019 */
-/* <O___,, * (see CREDITS file for the list of authors) */
+/* v * Copyright INRIA, CNRS and contributors */
+/* <O___,, * (see version control and CREDITS file for authors & dates) */
/* \VV/ **************************************************************/
/* // * This file is distributed under the terms of the */
/* * GNU Lesser General Public License Version 2.1 */
diff --git a/dev/header.ml b/dev/header.ml
index 87553dcb56..b72d544151 100644
--- a/dev/header.ml
+++ b/dev/header.ml
@@ -1,7 +1,7 @@
(************************************************************************)
(* * The Coq Proof Assistant / The Coq Development Team *)
-(* v * INRIA, CNRS and contributors - Copyright 1999-2019 *)
-(* <O___,, * (see CREDITS file for the list of authors) *)
+(* v * Copyright INRIA, CNRS and contributors *)
+(* <O___,, * (see version control and CREDITS file for authors & dates) *)
(* \VV/ **************************************************************)
(* // * This file is distributed under the terms of the *)
(* * GNU Lesser General Public License Version 2.1 *)
diff --git a/dev/header.py b/dev/header.py
index 86114503d4..2c39321f19 100644
--- a/dev/header.py
+++ b/dev/header.py
@@ -1,7 +1,7 @@
##########################################################################
## # The Coq Proof Assistant / The Coq Development Team ##
-## v # INRIA, CNRS and contributors - Copyright 1999-2019 ##
-## <O___,, # (see CREDITS file for the list of authors) ##
+## v # Copyright INRIA, CNRS and contributors ##
+## <O___,, # (see version control and CREDITS file for authors & dates) ##
## \VV/ ###############################################################
## // # This file is distributed under the terms of the ##
## # GNU Lesser General Public License Version 2.1 ##