diff -r b82e765ca464 -r df225aa45770 IntEx.thy --- a/IntEx.thy Wed Nov 04 09:52:31 2009 +0100 +++ b/IntEx.thy Wed Nov 04 10:31:20 2009 +0100 @@ -13,6 +13,7 @@ done print_theorems +print_quotients quotient_def ZERO::"my_int" @@ -38,18 +39,11 @@ quotient_def PLUS::"my_int \ my_int \ my_int" where - "PLUS \ my_plus" + "PLUS x y \ my_plus x y" term PLUS thm PLUS_def -definition - "MPLUS x y \ my_plus x y" - -term MPLUS -thm MPLUS_def -thm MPLUS_def_raw - fun my_neg :: "(nat \ nat) \ (nat \ nat)" where