author | paulson |
Mon, 19 Jul 1999 15:27:34 +0200 | |
changeset 7032 | d6efb3b8e669 |
child 9509 | 0f3ee1f89ca8 |
permissions | -rw-r--r-- |
7032 | 1 |
(* Title: HOL/NatBin.thy |
2 |
ID: $Id$ |
|
3 |
Author: Lawrence C Paulson, Cambridge University Computer Laboratory |
|
4 |
Copyright 1999 University of Cambridge |
|
5 |
||
6 |
Binary arithmetic for the natural numbers |
|
7 |
||
8 |
This case is simply reduced to that for the non-negative integers |
|
9 |
*) |
|
10 |
||
11 |
NatBin = IntDiv + |
|
12 |
||
13 |
instance |
|
14 |
nat :: number |
|
15 |
||
16 |
defs |
|
17 |
nat_number_of_def |
|
18 |
"number_of v == nat (number_of v)" |
|
19 |
(*::bin=>nat ::bin=>int*) |
|
20 |
||
21 |
end |