aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Ints/Int31.v
diff options
context:
space:
mode:
authorGravatar bgregoir <bgregoir@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-06-20 09:43:36 +0000
committerGravatar bgregoir <bgregoir@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-06-20 09:43:36 +0000
commitf4586d1e8b1116340574d9660117f93e7a1e4e3b (patch)
tree15b7dff4ed22b762446e4ae1f426e8f8aa2de52c /theories/Ints/Int31.v
parent4708506ca1b34e93835b163db102f6860c89190c (diff)
ajout de head0 et tail0 en natif
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@9900 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Ints/Int31.v')
-rw-r--r--theories/Ints/Int31.v5
1 files changed, 4 insertions, 1 deletions
diff --git a/theories/Ints/Int31.v b/theories/Ints/Int31.v
index 59e45c320..918c54232 100644
--- a/theories/Ints/Int31.v
+++ b/theories/Ints/Int31.v
@@ -402,4 +402,7 @@ Definition tail031 (i:int31) :=
| D1 => n
end)
i On
-. \ No newline at end of file
+.
+
+Register head031 as int31 head0 in "coq_int31" by True.
+Register tail031 as int31 tail0 in "coq_int31" by True.