aboutsummaryrefslogtreecommitdiffhomepage
path: root/plugins/dp
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-04-29 13:50:31 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-04-29 13:50:31 +0000
commitaf93e4cf8b1a839d21499b3b9737bb8904edcae8 (patch)
treeb9a4f28e6f8106bcf19e017f64147f836f810c4b /plugins/dp
parent0f61b02f84b41e1f019cd78824de28f18ff854aa (diff)
Remove the svn-specific $Id$ annotations
- Many of them were broken, some of them after Pierre B's rework of mli for ocamldoc, but not only (many bad annotation, many files with no svn property about Id, etc) - Useless for those of us that work with git-svn (and a fortiori in a forthcoming git-only setting) - Even in svn, they seem to be of little interest git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12972 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'plugins/dp')
-rw-r--r--plugins/dp/Dp.v2
-rw-r--r--plugins/dp/g_dp.ml42
-rw-r--r--plugins/dp/zenon.v2
3 files changed, 0 insertions, 6 deletions
diff --git a/plugins/dp/Dp.v b/plugins/dp/Dp.v
index bc7d73f62..1b66c334e 100644
--- a/plugins/dp/Dp.v
+++ b/plugins/dp/Dp.v
@@ -6,8 +6,6 @@ Require Export Classical.
(* Zenon *)
(* Copyright 2004 INRIA *)
-(* $Id$ *)
-
Lemma zenon_nottrue :
(~True -> False).
Proof. tauto. Qed.
diff --git a/plugins/dp/g_dp.ml4 b/plugins/dp/g_dp.ml4
index 82f86cd81..e2cd4b3e3 100644
--- a/plugins/dp/g_dp.ml4
+++ b/plugins/dp/g_dp.ml4
@@ -8,8 +8,6 @@
(*i camlp4deps: "parsing/grammar.cma" i*)
-(* $Id$ *)
-
open Dp
TACTIC EXTEND Simplify
diff --git a/plugins/dp/zenon.v b/plugins/dp/zenon.v
index 502465c6b..89028c4f4 100644
--- a/plugins/dp/zenon.v
+++ b/plugins/dp/zenon.v
@@ -1,6 +1,4 @@
(* Copyright 2004 INRIA *)
-(* $Id$ *)
-
Require Export Classical.
Lemma zenon_nottrue :