changeset 5078 | 7b5ea59c0275 |
child 5491 | 22f8331cdf47 |
--- /dev/null Thu Jan 01 00:00:00 1970 +0000 +++ b/src/HOL/ex/IntRingDefs.thy Thu Jun 25 13:57:34 1998 +0200 @@ -0,0 +1,15 @@ +(* Title: HOL/Integ/IntRingDefs.thy + ID: $Id$ + Author: Tobias Nipkow and Markus Wenzel + Copyright 1996 TU Muenchen + +Provides the basic defs and thms for showing that int is a commutative ring. +Most of it has been defined and shown already. +*) + +IntRingDefs = Integ + Ring + + +instance int :: zero +defs zero_int_def "zero::int == $# 0" + +end