src/HOL/NSA/CStar.thy
changeset 61975 b4b11391c676
parent 58878 f962e42e324d
child 61982 3af5a06577c7
--- a/src/HOL/NSA/CStar.thy	Wed Dec 30 11:32:56 2015 +0100
+++ b/src/HOL/NSA/CStar.thy	Wed Dec 30 11:37:29 2015 +0100
@@ -3,14 +3,14 @@
     Copyright   : 2001 University of Edinburgh
 *)
 
-section{*Star-transforms in NSA, Extending Sets of Complex Numbers
-      and Complex Functions*}
+section\<open>Star-transforms in NSA, Extending Sets of Complex Numbers
+      and Complex Functions\<close>
 
 theory CStar
 imports NSCA
 begin
 
-subsection{*Properties of the *-Transform Applied to Sets of Reals*}
+subsection\<open>Properties of the *-Transform Applied to Sets of Reals\<close>
 
 lemma STARC_hcomplex_of_complex_Int:
      "*s* X Int SComplex = hcomplex_of_complex ` X"
@@ -20,7 +20,7 @@
      "x \<notin> hcomplex_of_complex ` A ==> \<forall>y \<in> A. x \<noteq> hcomplex_of_complex y"
 by auto
 
-subsection{*Theorems about Nonstandard Extensions of Functions*}
+subsection\<open>Theorems about Nonstandard Extensions of Functions\<close>
 
 lemma starfunC_hcpow: "!!Z. ( *f* (%z. z ^ n)) Z = Z pow hypnat_of_nat n"
 by transfer (rule refl)
@@ -28,7 +28,7 @@
 lemma starfunCR_cmod: "*f* cmod = hcmod"
 by transfer (rule refl)
 
-subsection{*Internal Functions - Some Redundancy With *f* Now*}
+subsection\<open>Internal Functions - Some Redundancy With *f* Now\<close>
 
 (** subtraction: ( *fn) - ( *gn) = *(fn - gn) **)
 (*