author | oheimb |
Mon, 21 Sep 1998 23:25:27 +0200 | |
changeset 5526 | e7617b57a3e6 |
parent 5491 | 22f8331cdf47 |
child 5601 | b6456ccd9e3e |
permissions | -rw-r--r-- |
5078 | 1 |
(* Title: HOL/Integ/IntRingDefs.thy |
2 |
ID: $Id$ |
|
3 |
Author: Tobias Nipkow and Markus Wenzel |
|
4 |
Copyright 1996 TU Muenchen |
|
5 |
||
6 |
Provides the basic defs and thms for showing that int is a commutative ring. |
|
7 |
Most of it has been defined and shown already. |
|
8 |
*) |
|
9 |
||
5491 | 10 |
IntRingDefs = Main + Ring + |
5078 | 11 |
|
12 |
instance int :: zero |
|
5491 | 13 |
defs zero_int_def "zero::int == #0" |
5078 | 14 |
|
15 |
end |