aboutsummaryrefslogtreecommitdiffhomepage
path: root/plugins/setoid_ring/Algebra_syntax.v
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2018-03-30 12:16:23 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2018-03-30 15:12:53 +0200
commitf35a68f6b01fdd167f712bd9a0df0154225497b9 (patch)
tree0df6a724677efe3c716f18bbc4319958a9bb14b1 /plugins/setoid_ring/Algebra_syntax.v
parentbd8606189268c3fcdd3506872d459cb9032a33bf (diff)
Adding some headers, by consistency of style.
[skip ci]
Diffstat (limited to 'plugins/setoid_ring/Algebra_syntax.v')
-rw-r--r--plugins/setoid_ring/Algebra_syntax.v9
1 files changed, 9 insertions, 0 deletions
diff --git a/plugins/setoid_ring/Algebra_syntax.v b/plugins/setoid_ring/Algebra_syntax.v
index e896554ea..1204bbd2e 100644
--- a/plugins/setoid_ring/Algebra_syntax.v
+++ b/plugins/setoid_ring/Algebra_syntax.v
@@ -1,3 +1,12 @@
+(************************************************************************)
+(* * 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) *)
+(************************************************************************)
Class Zero (A : Type) := zero : A.
Notation "0" := zero.