src/HOL/Complex/NSComplex.thy
changeset 14653 0848ab6fe5fc
parent 14641 79b7bd936264
child 14658 b1293d0f8d5f
--- a/src/HOL/Complex/NSComplex.thy	Thu Apr 22 11:02:22 2004 +0200
+++ b/src/HOL/Complex/NSComplex.thy	Thu Apr 22 12:11:17 2004 +0200
@@ -86,16 +86,16 @@
   hcis :: "hypreal => hcomplex"
   "hcis a == Abs_hcomplex(UN X:Rep_hypreal(a). hcomplexrel `` {%n. cis (X n)})"
 
-  (* abbreviation for r*(cos a + i sin a) *)
-  hrcis :: "[hypreal, hypreal] => hcomplex"
-  "hrcis r a == hcomplex_of_hypreal r * hcis a"
-
   (*----- injection from hyperreals -----*)
 
   hcomplex_of_hypreal :: "hypreal => hcomplex"
   "hcomplex_of_hypreal r == Abs_hcomplex(UN X:Rep_hypreal(r).
 			       hcomplexrel `` {%n. complex_of_real (X n)})"
 
+  (* abbreviation for r*(cos a + i sin a) *)
+  hrcis :: "[hypreal, hypreal] => hcomplex"
+  "hrcis r a == hcomplex_of_hypreal r * hcis a"
+
   (*------------ e ^ (x + iy) ------------*)
 
   hexpi :: "hcomplex => hcomplex"