aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/IntMap
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-11-12 16:25:16 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-11-12 16:25:16 +0000
commitea9f6b8f620b9f69de9d72ca603af042e4487339 (patch)
treeca67e410a2f0de981e4f1ed2aba109068ea61d29 /theories/IntMap
parent6931f2b04580fb088fa9c4a09129e77dad3f387c (diff)
On sait jamais
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4862 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/IntMap')
-rw-r--r--theories/IntMap/Adalloc.v6
1 files changed, 6 insertions, 0 deletions
diff --git a/theories/IntMap/Adalloc.v b/theories/IntMap/Adalloc.v
index d2ca86b2f..5dcd41c84 100644
--- a/theories/IntMap/Adalloc.v
+++ b/theories/IntMap/Adalloc.v
@@ -331,3 +331,9 @@ Section AdAlloc.
Qed.
End AdAlloc.
+
+V7only [
+(* Moved to NArith *)
+Notation positive_to_nat_2 := positive_to_nat_2.
+Notation positive_to_nat_4 := positive_to_nat_4.
+].