src/HOL/Integ/IntDef.thy
changeset 11701 3d51fbf81c17
parent 11451 8abfb4f7bd02
child 11713 883d559b0b8c
equal deleted inserted replaced
11700:a0e6bda62b7b 11701:3d51fbf81c17
    33   iszero :: int => bool
    33   iszero :: int => bool
    34   "iszero z == z = int 0"
    34   "iszero z == z = int 0"
    35   
    35   
    36 defs (*of overloaded constants*)
    36 defs (*of overloaded constants*)
    37   
    37   
    38   Zero_def      "0 == int 0"
    38   Zero_int_def      "0 == int 0"
    39 
    39 
    40   zadd_def
    40   zadd_def
    41    "z + w == 
    41    "z + w == 
    42        Abs_Integ(UN (x1,y1):Rep_Integ(z). UN (x2,y2):Rep_Integ(w).   
    42        Abs_Integ(UN (x1,y1):Rep_Integ(z). UN (x2,y2):Rep_Integ(w).   
    43 		 intrel``{(x1+x2, y1+y2)})"
    43 		 intrel``{(x1+x2, y1+y2)})"