aboutsummaryrefslogtreecommitdiffhomepage
path: root/lib
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-04-01 14:45:20 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-04-01 14:45:20 +0000
commit124016815a5a38dfebee75451721ae13bca81959 (patch)
treeb3adc59b7ecc5fb6093e21a741bf764fa206864f /lib
parent97fb9f22eadab06fe320ccedf6abfb6be89702f4 (diff)
Ajout des propriétés $Id:$ là où elles n'existaient pas ou n'étaient
pas correctes git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10739 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'lib')
-rw-r--r--lib/flags.ml2
-rw-r--r--lib/flags.mli2
-rw-r--r--lib/option.ml2
3 files changed, 3 insertions, 3 deletions
diff --git a/lib/flags.ml b/lib/flags.ml
index 12b2ed037..6a801480a 100644
--- a/lib/flags.ml
+++ b/lib/flags.ml
@@ -6,7 +6,7 @@
(* * GNU Lesser General Public License Version 2.1 *)
(************************************************************************)
-(* $Id: options.ml 10106 2007-08-30 16:56:10Z herbelin $ *)
+(*i $Id:$ i*)
open Util
diff --git a/lib/flags.mli b/lib/flags.mli
index 248b59b0d..73962735d 100644
--- a/lib/flags.mli
+++ b/lib/flags.mli
@@ -6,7 +6,7 @@
(* * GNU Lesser General Public License Version 2.1 *)
(************************************************************************)
-(*i $Id: options.mli 9679 2007-02-24 15:22:07Z herbelin $ i*)
+(*i $Id$ i*)
(* Global options of the system. *)
diff --git a/lib/option.ml b/lib/option.ml
index 95a18396b..543c108ab 100644
--- a/lib/option.ml
+++ b/lib/option.ml
@@ -6,7 +6,7 @@
(* * GNU Lesser General Public License Version 2.1 *)
(************************************************************************)
-(* $Id$ *)
+(*i $Id:$ i*)
(** Module implementing basic combinators for OCaml option type.
It tries follow closely the style of OCaml standard library.