src/HOL/Integ/IntDef.thy
author berghofe
Fri, 19 Apr 2002 14:33:04 +0200
changeset 13089 c8c28a1dc787
parent 11868 56db9f3a6b3e
child 13487 1291c6375c29
permissions -rw-r--r--
Added proof of Newman's lemma.
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
5508
691c70898518 new files in Integ
paulson
parents:
diff changeset
     1
(*  Title:      IntDef.thy
691c70898518 new files in Integ
paulson
parents:
diff changeset
     2
    ID:         $Id$
691c70898518 new files in Integ
paulson
parents:
diff changeset
     3
    Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
691c70898518 new files in Integ
paulson
parents:
diff changeset
     4
    Copyright   1996  University of Cambridge
691c70898518 new files in Integ
paulson
parents:
diff changeset
     5
691c70898518 new files in Integ
paulson
parents:
diff changeset
     6
The integers as equivalence classes over nat*nat.
691c70898518 new files in Integ
paulson
parents:
diff changeset
     7
*)
691c70898518 new files in Integ
paulson
parents:
diff changeset
     8
11451
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents: 10834
diff changeset
     9
IntDef = Equiv + NatArith + 
5508
691c70898518 new files in Integ
paulson
parents:
diff changeset
    10
constdefs
691c70898518 new files in Integ
paulson
parents:
diff changeset
    11
  intrel      :: "((nat * nat) * (nat * nat)) set"
9392
c8e6529cc082 changed / to // for quotienting
paulson
parents: 8937
diff changeset
    12
  "intrel == {p. EX x1 y1 x2 y2. p=((x1::nat,y1),(x2,y2)) & x1+y2 = x2+y1}"
5508
691c70898518 new files in Integ
paulson
parents:
diff changeset
    13
691c70898518 new files in Integ
paulson
parents:
diff changeset
    14
typedef (Integ)
9392
c8e6529cc082 changed / to // for quotienting
paulson
parents: 8937
diff changeset
    15
  int = "UNIV//intrel"            (Equiv.quotient_def)
5508
691c70898518 new files in Integ
paulson
parents:
diff changeset
    16
691c70898518 new files in Integ
paulson
parents:
diff changeset
    17
instance
11713
883d559b0b8c sane numerals (stage 3): provide generic "1" on all number types;
wenzelm
parents: 11701
diff changeset
    18
  int :: {ord, zero, one, plus, times, minus}
5508
691c70898518 new files in Integ
paulson
parents:
diff changeset
    19
691c70898518 new files in Integ
paulson
parents:
diff changeset
    20
defs
691c70898518 new files in Integ
paulson
parents:
diff changeset
    21
  zminus_def
10834
a7897aebbffc *** empty log message ***
nipkow
parents: 10797
diff changeset
    22
    "- Z == Abs_Integ(UN (x,y):Rep_Integ(Z). intrel``{(y,x)})"
5508
691c70898518 new files in Integ
paulson
parents:
diff changeset
    23
691c70898518 new files in Integ
paulson
parents:
diff changeset
    24
constdefs
691c70898518 new files in Integ
paulson
parents:
diff changeset
    25
5582
a356fb49e69e many renamings and changes. Simproc for cancelling common terms in relations
paulson
parents: 5562
diff changeset
    26
  int :: nat => int
10834
a7897aebbffc *** empty log message ***
nipkow
parents: 10797
diff changeset
    27
  "int m == Abs_Integ(intrel `` {(m,0)})"
5508
691c70898518 new files in Integ
paulson
parents:
diff changeset
    28
5540
0f16c3b66ab4 much renaming and reorganization
paulson
parents: 5508
diff changeset
    29
  neg   :: int => bool
0f16c3b66ab4 much renaming and reorganization
paulson
parents: 5508
diff changeset
    30
  "neg(Z) == EX x y. x<y & (x,y::nat):Rep_Integ(Z)"
5508
691c70898518 new files in Integ
paulson
parents:
diff changeset
    31
691c70898518 new files in Integ
paulson
parents:
diff changeset
    32
  (*For simplifying equalities*)
691c70898518 new files in Integ
paulson
parents:
diff changeset
    33
  iszero :: int => bool
11868
56db9f3a6b3e Numerals now work for the integers: the binary numerals for 0 and 1 rewrite
paulson
parents: 11713
diff changeset
    34
  "iszero z == z = (0::int)"
5508
691c70898518 new files in Integ
paulson
parents:
diff changeset
    35
  
9392
c8e6529cc082 changed / to // for quotienting
paulson
parents: 8937
diff changeset
    36
defs (*of overloaded constants*)
c8e6529cc082 changed / to // for quotienting
paulson
parents: 8937
diff changeset
    37
  
11713
883d559b0b8c sane numerals (stage 3): provide generic "1" on all number types;
wenzelm
parents: 11701
diff changeset
    38
  Zero_int_def "0 == int 0"
883d559b0b8c sane numerals (stage 3): provide generic "1" on all number types;
wenzelm
parents: 11701
diff changeset
    39
  One_int_def "1 == int 1"
8937
7328d7c8d201 defining 0::int to be (int 0)
paulson
parents: 7375
diff changeset
    40
5508
691c70898518 new files in Integ
paulson
parents:
diff changeset
    41
  zadd_def
5594
e4439230af67 much tidying
paulson
parents: 5582
diff changeset
    42
   "z + w == 
7375
2cb340e66d15 tidied, allowing pattern-matching in defs of zadd and zmult
paulson
parents: 7127
diff changeset
    43
       Abs_Integ(UN (x1,y1):Rep_Integ(z). UN (x2,y2):Rep_Integ(w).   
10834
a7897aebbffc *** empty log message ***
nipkow
parents: 10797
diff changeset
    44
		 intrel``{(x1+x2, y1+y2)})"
5508
691c70898518 new files in Integ
paulson
parents:
diff changeset
    45
7127
48e235179ffb added parentheses to cope with a possible reduction of the precedence of unary
paulson
parents: 5594
diff changeset
    46
  zdiff_def "z - (w::int) == z + (-w)"
5508
691c70898518 new files in Integ
paulson
parents:
diff changeset
    47
5594
e4439230af67 much tidying
paulson
parents: 5582
diff changeset
    48
  zless_def "z<w == neg(z - w)"
5508
691c70898518 new files in Integ
paulson
parents:
diff changeset
    49
5594
e4439230af67 much tidying
paulson
parents: 5582
diff changeset
    50
  zle_def   "z <= (w::int) == ~(w < z)"
5508
691c70898518 new files in Integ
paulson
parents:
diff changeset
    51
691c70898518 new files in Integ
paulson
parents:
diff changeset
    52
  zmult_def
5594
e4439230af67 much tidying
paulson
parents: 5582
diff changeset
    53
   "z * w == 
7375
2cb340e66d15 tidied, allowing pattern-matching in defs of zadd and zmult
paulson
parents: 7127
diff changeset
    54
       Abs_Integ(UN (x1,y1):Rep_Integ(z). UN (x2,y2):Rep_Integ(w).   
10834
a7897aebbffc *** empty log message ***
nipkow
parents: 10797
diff changeset
    55
		 intrel``{(x1*x2 + y1*y2, x1*y2 + y1*x2)})"
5508
691c70898518 new files in Integ
paulson
parents:
diff changeset
    56
691c70898518 new files in Integ
paulson
parents:
diff changeset
    57
end