aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics
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 /tactics
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 'tactics')
-rw-r--r--tactics/class_tactics.ml42
-rw-r--r--tactics/decl_interp.ml2
2 files changed, 2 insertions, 2 deletions
diff --git a/tactics/class_tactics.ml4 b/tactics/class_tactics.ml4
index 6a8d0d36d..5c2422477 100644
--- a/tactics/class_tactics.ml4
+++ b/tactics/class_tactics.ml4
@@ -9,7 +9,7 @@
(*i camlp4deps: "parsing/grammar.cma" i*)
-(* $Id: eauto.ml4 10346 2007-12-05 21:11:19Z aspiwack $ *)
+(* $Id$ *)
open Pp
open Util
diff --git a/tactics/decl_interp.ml b/tactics/decl_interp.ml
index b33fbde8a..4eb59a2fb 100644
--- a/tactics/decl_interp.ml
+++ b/tactics/decl_interp.ml
@@ -6,7 +6,7 @@
(* * GNU Lesser General Public License Version 2.1 *)
(************************************************************************)
-(* $Id$ *)
+(*i $Id:$ i*)
open Util
open Names