src/HOL/ex/IntRingDefs.ML
changeset 8936 a1c426541757
parent 8935 548901d05a0e
child 8937 7328d7c8d201
equal deleted inserted replaced
8935:548901d05a0e 8936:a1c426541757
     1 (*  Title:      HOL/ex/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";