src/HOL/Complex/ComplexBin.thy
author kleing
Tue, 13 May 2003 08:59:21 +0200
changeset 14024 213dcc39358f
parent 13957 10dbf16be15f
child 14387 e96d5c42c4b0
permissions -rw-r--r--
HOL-Real -> HOL-Complex
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
13957
10dbf16be15f new session Complex for the complex numbers
paulson
parents:
diff changeset
     1
(*  Title:      ComplexBin.thy
10dbf16be15f new session Complex for the complex numbers
paulson
parents:
diff changeset
     2
    Author:     Jacques D. Fleuriot
10dbf16be15f new session Complex for the complex numbers
paulson
parents:
diff changeset
     3
    Copyright:  2001 University of Edinburgh
10dbf16be15f new session Complex for the complex numbers
paulson
parents:
diff changeset
     4
    Descrition: Binary arithmetic for the complex numbers
10dbf16be15f new session Complex for the complex numbers
paulson
parents:
diff changeset
     5
                This case is reduced to that for the reals.
10dbf16be15f new session Complex for the complex numbers
paulson
parents:
diff changeset
     6
*)
10dbf16be15f new session Complex for the complex numbers
paulson
parents:
diff changeset
     7
10dbf16be15f new session Complex for the complex numbers
paulson
parents:
diff changeset
     8
ComplexBin = Complex + 
10dbf16be15f new session Complex for the complex numbers
paulson
parents:
diff changeset
     9
10dbf16be15f new session Complex for the complex numbers
paulson
parents:
diff changeset
    10
10dbf16be15f new session Complex for the complex numbers
paulson
parents:
diff changeset
    11
instance
10dbf16be15f new session Complex for the complex numbers
paulson
parents:
diff changeset
    12
  complex :: number 
10dbf16be15f new session Complex for the complex numbers
paulson
parents:
diff changeset
    13
10dbf16be15f new session Complex for the complex numbers
paulson
parents:
diff changeset
    14
instance complex :: plus_ac0(complex_add_commute,complex_add_assoc,complex_add_zero_left)
10dbf16be15f new session Complex for the complex numbers
paulson
parents:
diff changeset
    15
10dbf16be15f new session Complex for the complex numbers
paulson
parents:
diff changeset
    16
10dbf16be15f new session Complex for the complex numbers
paulson
parents:
diff changeset
    17
defs
10dbf16be15f new session Complex for the complex numbers
paulson
parents:
diff changeset
    18
  complex_number_of_def
10dbf16be15f new session Complex for the complex numbers
paulson
parents:
diff changeset
    19
    "number_of v == complex_of_real (number_of v)"
10dbf16be15f new session Complex for the complex numbers
paulson
parents:
diff changeset
    20
     (*::bin=>complex               ::bin=>complex*)
10dbf16be15f new session Complex for the complex numbers
paulson
parents:
diff changeset
    21
10dbf16be15f new session Complex for the complex numbers
paulson
parents:
diff changeset
    22
end