src/HOL/Complex/NSComplexBin.thy
changeset 13957 10dbf16be15f
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/src/HOL/Complex/NSComplexBin.thy	Mon May 05 18:22:31 2003 +0200
@@ -0,0 +1,19 @@
+(*  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
\ No newline at end of file