src/HOL/ex/IntRingDefs.ML
author wenzelm
Thu, 30 Sep 1999 21:21:04 +0200
changeset 7664 c151ac595551
parent 5601 b6456ccd9e3e
permissions -rw-r--r--
insert: ignore facts;

(*  Title:      HOL/ex/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";