author | paulson |
Wed, 05 Aug 1998 10:57:25 +0200 | |
changeset 5253 | 82a5ca6290aa |
parent 5227 | e5a6ace920a0 |
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 |
||
7 |
Goalw [zero_int_def,zdiff_def] "(zero-x)+(x::int) = zero"; |
|
8 |
by (Simp_tac 1); |
|
9 |
qed "left_inv_int"; |
|
10 |
||
11 |
Goalw [zero_int_def,zdiff_def] "x-y = (x::int) + (zero-y)"; |
|
12 |
by (Simp_tac 1); |
|
13 |
qed "minus_inv_int"; |