| author | wenzelm |
| Thu, 16 Oct 1997 13:33:17 +0200 | |
| changeset 3884 | 5423e06b9fe6 |
| parent 3370 | 5c5fdce3a4e4 |
| child 4104 | 84433b1ab826 |
| permissions | -rw-r--r-- |
| 923 | 1 |
(* Title: HOL/Nat.thy |
2 |
ID: $Id$ |
|
| 2608 | 3 |
Author: Tobias Nipkow |
4 |
Copyright 1997 TU Muenchen |
|
| 923 | 5 |
|
| 2608 | 6 |
Nat is a partial order |
| 923 | 7 |
*) |
8 |
||
| 2608 | 9 |
Nat = NatDef + |
| 923 | 10 |
|
| 2608 | 11 |
instance nat :: order (le_refl,le_trans,le_anti_sym,nat_less_le) |
| 1660 | 12 |
|
|
3370
5c5fdce3a4e4
Overloading of "^" requires new type class "power", with types "nat" and
paulson
parents:
2608
diff
changeset
|
13 |
consts |
|
5c5fdce3a4e4
Overloading of "^" requires new type class "power", with types "nat" and
paulson
parents:
2608
diff
changeset
|
14 |
"^" :: ['a::power,nat] => 'a (infixr 80) |
|
5c5fdce3a4e4
Overloading of "^" requires new type class "power", with types "nat" and
paulson
parents:
2608
diff
changeset
|
15 |
|
| 923 | 16 |
end |