aboutsummaryrefslogtreecommitdiff
path: root/plugins
diff options
context:
space:
mode:
authorThéo Zimmermann2019-02-06 09:31:42 +0100
committerThéo Zimmermann2019-02-06 09:31:42 +0100
commitb7b938a6878b754089814cbfdd478d6b9380c6bb (patch)
tree5681ea6302ceaffb8e8b2f715d73aebced91348a /plugins
parentd9afe70c9c65359b6eb827f5b30d84f24074efa1 (diff)
Fix #9281: forgotten CeCILL-B headers in ssrmatching plugin.
Diffstat (limited to 'plugins')
-rw-r--r--plugins/ssrmatching/g_ssrmatching.mlg2
-rw-r--r--plugins/ssrmatching/g_ssrmatching.mli13
2 files changed, 13 insertions, 2 deletions
diff --git a/plugins/ssrmatching/g_ssrmatching.mlg b/plugins/ssrmatching/g_ssrmatching.mlg
index 4ddaeb49fd..d1c7a23e99 100644
--- a/plugins/ssrmatching/g_ssrmatching.mlg
+++ b/plugins/ssrmatching/g_ssrmatching.mlg
@@ -8,6 +8,8 @@
(* * (see LICENSE file for the text of the license) *)
(************************************************************************)
+(* (c) Copyright 2006-2015 Microsoft Corporation and Inria. *)
+
{
open Ltac_plugin
diff --git a/plugins/ssrmatching/g_ssrmatching.mli b/plugins/ssrmatching/g_ssrmatching.mli
index 588a1a3eac..65ea3f79c8 100644
--- a/plugins/ssrmatching/g_ssrmatching.mli
+++ b/plugins/ssrmatching/g_ssrmatching.mli
@@ -1,5 +1,14 @@
-(* (c) Copyright 2006-2015 Microsoft Corporation and Inria. *)
-(* Distributed under the terms of CeCILL-B. *)
+(************************************************************************)
+(* * 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) *)
+(************************************************************************)
+
+(* (c) Copyright 2006-2015 Microsoft Corporation and Inria. *)
open Genarg
open Ssrmatching