diff -r 93c9022ba5e9 -r c4001cda9da3 Quot/Examples/IntEx2.thy --- a/Quot/Examples/IntEx2.thy Fri Feb 12 15:50:43 2010 +0100 +++ b/Quot/Examples/IntEx2.thy Fri Feb 12 16:04:10 2010 +0100 @@ -21,10 +21,10 @@ ML {* @{term "0 \ int"} *} quotient_definition - "0 \ int" as "(0\nat, 0\nat)" + "0 \ int" is "(0\nat, 0\nat)" quotient_definition - "1 \ int" as "(1\nat, 0\nat)" + "1 \ int" is "(1\nat, 0\nat)" fun plus_raw :: "(nat \ nat) \ (nat \ nat) \ (nat \ nat)" @@ -32,7 +32,7 @@ "plus_raw (x, y) (u, v) = (x + u, y + v)" quotient_definition - "(op +) \ (int \ int \ int)" as "plus_raw" + "(op +) \ (int \ int \ int)" is "plus_raw" fun uminus_raw :: "(nat \ nat) \ (nat \ nat)" @@ -40,7 +40,7 @@ "uminus_raw (x, y) = (y, x)" quotient_definition - "(uminus \ (int \ int))" as "uminus_raw" + "(uminus \ (int \ int))" is "uminus_raw" definition minus_int_def [code del]: "z - w = z + (-w\int)" @@ -51,7 +51,7 @@ "mult_raw (x, y) (u, v) = (x*u + y*v, x*v + y*u)" quotient_definition - mult_int_def: "(op *) :: (int \ int \ int)" as "mult_raw" + mult_int_def: "(op *) :: (int \ int \ int)" is "mult_raw" fun le_raw :: "(nat \ nat) \ (nat \ nat) \ bool" @@ -59,7 +59,7 @@ "le_raw (x, y) (u, v) = (x+v \ u+y)" quotient_definition - le_int_def: "(op \) :: int \ int \ bool" as "le_raw" + le_int_def: "(op \) :: int \ int \ bool" is "le_raw" definition less_int_def [code del]: "(z\int) < w = (z \ w \ z \ w)" @@ -207,7 +207,7 @@ "int_of_nat_raw m = (m :: nat, 0 :: nat)" quotient_definition - "int_of_nat :: nat \ int" as "int_of_nat_raw" + "int_of_nat :: nat \ int" is "int_of_nat_raw" lemma[quot_respect]: shows "(op = ===> op \) int_of_nat_raw int_of_nat_raw"