diff -r 3764566c1151 -r 4d58c02289ca IntEx.thy --- a/IntEx.thy Tue Nov 03 16:17:19 2009 +0100 +++ b/IntEx.thy Tue Nov 03 16:51:33 2009 +0100 @@ -14,13 +14,15 @@ print_theorems -quotient_def (for my_int) +quotient_def ZERO::"my_int" where "ZERO \ (0::nat, 0::nat)" +term ZERO +thm ZERO_def -quotient_def (for my_int) +quotient_def ONE::"my_int" where "ONE \ (1::nat, 0::nat)" @@ -33,7 +35,7 @@ where "my_plus (x, y) (u, v) = (x + u, y + v)" -quotient_def (for my_int) +quotient_def PLUS::"my_int \ my_int \ my_int" where "PLUS \ my_plus" @@ -48,13 +50,12 @@ thm MPLUS_def thm MPLUS_def_raw - fun my_neg :: "(nat \ nat) \ (nat \ nat)" where "my_neg (x, y) = (y, x)" -quotient_def (for my_int) +quotient_def NEG::"my_int \ my_int" where "NEG \ my_neg" @@ -72,7 +73,7 @@ where "my_mult (x, y) (u, v) = (x*u + y*v, x*v + y*u)" -quotient_def (for my_int) +quotient_def MULT::"my_int \ my_int \ my_int" where "MULT \ my_mult" @@ -86,7 +87,7 @@ where "my_le (x, y) (u, v) = (x+v \ u+y)" -quotient_def (for my_int) +quotient_def LE :: "my_int \ my_int \ bool" where "LE \ my_le"