diff -r df053507edba -r 37285ec4387d Quot/Examples/LarryInt.thy --- a/Quot/Examples/LarryInt.thy Sun Dec 20 00:26:53 2009 +0100 +++ b/Quot/Examples/LarryInt.thy Sun Dec 20 00:53:35 2009 +0100 @@ -16,16 +16,16 @@ instantiation int :: "{zero, one, plus, uminus, minus, times, ord}" begin -quotient_def +quotient_definition Zero_int_def: "0::int" as "(0::nat, 0::nat)" -quotient_def +quotient_definition One_int_def: "1::int" as "(1::nat, 0::nat)" definition "add_raw \ \(x, y) (u, v). (x + (u::nat), y + (v::nat))" -quotient_def +quotient_definition "(op +) :: int \ int \ int" as "add_raw" @@ -33,7 +33,7 @@ definition "uminus_raw \ \(x::nat, y::nat). (y, x)" -quotient_def +quotient_definition "uminus :: int \ int" as "uminus_raw" @@ -43,7 +43,7 @@ where "mult_raw (x, y) (u, v) = (x*u + y*v, x*v + y*u)" -quotient_def +quotient_definition "(op *) :: int \ int \ int" as "mult_raw" @@ -51,7 +51,7 @@ definition "le_raw \ \(x, y) (u, v). (x+v \ u+(y::nat))" -quotient_def +quotient_definition le_int_def: "(op \) :: int \ int \ bool" as "le_raw" @@ -343,7 +343,7 @@ definition "nat_raw \ \(x, y).x - (y::nat)" -quotient_def +quotient_definition "nat2::int\nat" as "nat_raw"