aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/NArith
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 /theories/NArith
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 'theories/NArith')
-rw-r--r--theories/NArith/BinNat.v2
-rw-r--r--theories/NArith/BinPos.v2
-rw-r--r--theories/NArith/NArith.v2
-rw-r--r--theories/NArith/Ndec.v2
-rw-r--r--theories/NArith/Ndigits.v2
-rw-r--r--theories/NArith/Ndist.v2
-rw-r--r--theories/NArith/Nnat.v2
-rw-r--r--theories/NArith/Pnat.v2
8 files changed, 0 insertions, 16 deletions
diff --git a/theories/NArith/BinNat.v b/theories/NArith/BinNat.v
index b289380fd..6b668df60 100644
--- a/theories/NArith/BinNat.v
+++ b/theories/NArith/BinNat.v
@@ -6,8 +6,6 @@
(* * GNU Lesser General Public License Version 2.1 *)
(************************************************************************)
-(*i $Id$ i*)
-
Require Import BinPos.
Unset Boxed Definitions.
diff --git a/theories/NArith/BinPos.v b/theories/NArith/BinPos.v
index a5f99cc66..a7b2336c8 100644
--- a/theories/NArith/BinPos.v
+++ b/theories/NArith/BinPos.v
@@ -7,8 +7,6 @@
(* * GNU Lesser General Public License Version 2.1 *)
(************************************************************************)
-(*i $Id$ i*)
-
Unset Boxed Definitions.
Declare ML Module "z_syntax_plugin".
diff --git a/theories/NArith/NArith.v b/theories/NArith/NArith.v
index 009e64fd0..7282fc758 100644
--- a/theories/NArith/NArith.v
+++ b/theories/NArith/NArith.v
@@ -6,8 +6,6 @@
(* * GNU Lesser General Public License Version 2.1 *)
(************************************************************************)
-(* $Id$ *)
-
(** Library for binary natural numbers *)
Require Export BinPos.
diff --git a/theories/NArith/Ndec.v b/theories/NArith/Ndec.v
index 9540aace7..c217ada11 100644
--- a/theories/NArith/Ndec.v
+++ b/theories/NArith/Ndec.v
@@ -6,8 +6,6 @@
(* * GNU Lesser General Public License Version 2.1 *)
(************************************************************************)
-(*i $Id$ i*)
-
Require Import Bool.
Require Import Sumbool.
Require Import Arith.
diff --git a/theories/NArith/Ndigits.v b/theories/NArith/Ndigits.v
index b699b7428..a79cfac3d 100644
--- a/theories/NArith/Ndigits.v
+++ b/theories/NArith/Ndigits.v
@@ -6,8 +6,6 @@
(* * GNU Lesser General Public License Version 2.1 *)
(************************************************************************)
-(*i $Id$ i*)
-
Require Import Bool Setoid Bvector BinPos BinNat.
(** Operation over bits of a [N] number. *)
diff --git a/theories/NArith/Ndist.v b/theories/NArith/Ndist.v
index 92559ff67..dc37fa6c2 100644
--- a/theories/NArith/Ndist.v
+++ b/theories/NArith/Ndist.v
@@ -5,8 +5,6 @@
(* // * This file is distributed under the terms of the *)
(* * GNU Lesser General Public License Version 2.1 *)
(************************************************************************)
-(*i $Id$ i*)
-
Require Import Arith.
Require Import Min.
Require Import BinPos.
diff --git a/theories/NArith/Nnat.v b/theories/NArith/Nnat.v
index 0016d035f..feabd3b16 100644
--- a/theories/NArith/Nnat.v
+++ b/theories/NArith/Nnat.v
@@ -6,8 +6,6 @@
(* * GNU Lesser General Public License Version 2.1 *)
(************************************************************************)
-(*i $Id$ i*)
-
Require Import Arith_base.
Require Import Compare_dec.
Require Import Sumbool.
diff --git a/theories/NArith/Pnat.v b/theories/NArith/Pnat.v
index 0891dea21..fea12a1d4 100644
--- a/theories/NArith/Pnat.v
+++ b/theories/NArith/Pnat.v
@@ -7,8 +7,6 @@
(* * GNU Lesser General Public License Version 2.1 *)
(************************************************************************)
-(*i $Id$ i*)
-
Require Import BinPos.
(**********************************************************************)