diff options
author | Maxime Dénès <mail@maximedenes.fr> | 2018-03-05 13:30:08 +0100 |
---|---|---|
committer | Maxime Dénès <mail@maximedenes.fr> | 2018-03-05 13:30:08 +0100 |
commit | 15331729aaab16678c2f7e29dd391f72df53d76e (patch) | |
tree | 259c87baa8152c7b67fd339bb90f5ecf6317c207 /theories/Structures/Equalities.v | |
parent | 736e86e06b5831a0dd4b6a655708b4ffd2b4ee64 (diff) | |
parent | 629fbc743f8b5e7623a6834f19885b2e379cb782 (diff) |
Merge PR #6855: Update headers following #6543.
Diffstat (limited to 'theories/Structures/Equalities.v')
-rw-r--r-- | theories/Structures/Equalities.v | 16 |
1 files changed, 9 insertions, 7 deletions
diff --git a/theories/Structures/Equalities.v b/theories/Structures/Equalities.v index 747d03f8a..5f60a979c 100644 --- a/theories/Structures/Equalities.v +++ b/theories/Structures/Equalities.v @@ -1,10 +1,12 @@ -(***********************************************************************) -(* 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 *) -(***********************************************************************) +(************************************************************************) +(* * The Coq Proof Assistant / The Coq Development Team *) +(* v * INRIA, CNRS and contributors - Copyright 1999-2018 *) +(* <O___,, * (see CREDITS file for the list of authors) *) +(* \VV/ **************************************************************) +(* // * This file is distributed under the terms of the *) +(* * GNU Lesser General Public License Version 2.1 *) +(* * (see LICENSE file for the text of the license) *) +(************************************************************************) Require Export RelationClasses. Require Import Bool Morphisms Setoid. |