src/HOL/Complex/NSComplexBin.thy
author paulson
Fri, 15 Aug 2003 13:45:39 +0200
changeset 14151 b8bb6a6a2c46
parent 13957 10dbf16be15f
permissions -rw-r--r--
converting ex/If to Isar script

(*  Title:      NSComplexBin.thy
    Author:     Jacques D. Fleuriot
    Copyright:  2001 University of Edinburgh
    Descrition: Binary arithmetic for the nonstandard complex numbers
                This case is reduced to that for the complexes (hence reals).
*)

NSComplexBin = NSComplex + 


instance
  hcomplex :: number 

defs
  hcomplex_number_of_def
    "number_of v == hcomplex_of_complex (number_of v)"
     (*::bin=>complex               ::bin=>complex*)

end