author | paulson |
Wed, 05 Aug 1998 10:57:25 +0200 | |
changeset 5253 | 82a5ca6290aa |
parent 5227 | e5a6ace920a0 |
child 5601 | b6456ccd9e3e |
permissions | -rw-r--r-- |
(* Title: HOL/Integ/IntRingDefs.thy ID: $Id$ Author: Tobias Nipkow and Markus Wenzel Copyright 1996 TU Muenchen *) Goalw [zero_int_def,zdiff_def] "(zero-x)+(x::int) = zero"; by (Simp_tac 1); qed "left_inv_int"; Goalw [zero_int_def,zdiff_def] "x-y = (x::int) + (zero-y)"; by (Simp_tac 1); qed "minus_inv_int";