src/HOL/Integ/Integ.thy
author paulson
Fri, 18 Sep 1998 16:04:44 +0200
changeset 5509 c38cc427976c
parent 5491 22f8331cdf47
child 5540 0f16c3b66ab4
permissions -rw-r--r--
Now defines "int" as a linear order; basic derivations moved to IntDef

(*  Title:      Integ.thy
    ID:         $Id$
    Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
    Copyright   1998  University of Cambridge

Type "int" is a linear order
*)

Integ = IntDef +

instance int :: order (zle_refl,zle_trans,zle_anti_sym,int_less_le)
instance int :: linorder (zle_linear)

constdefs
  zmagnitude  :: int => nat
  "zmagnitude(Z) == @m. Z = $# m | -Z = $# m"

end