| author | paulson | 
| Thu, 04 Sep 2003 11:15:53 +0200 | |
| changeset 14182 | 5f49f00fe084 | 
| parent 13957 | 10dbf16be15f | 
| child 14387 | e96d5c42c4b0 | 
| permissions | -rw-r--r-- | 
(* Title: ComplexBin.thy Author: Jacques D. Fleuriot Copyright: 2001 University of Edinburgh Descrition: Binary arithmetic for the complex numbers This case is reduced to that for the reals. *) ComplexBin = Complex + instance complex :: number instance complex :: plus_ac0(complex_add_commute,complex_add_assoc,complex_add_zero_left) defs complex_number_of_def "number_of v == complex_of_real (number_of v)" (*::bin=>complex ::bin=>complex*) end