src/HOL/Complex.thy
changeset 61799 4cf66f21b764
parent 61762 d50b993b4fb9
child 61848 9250e546ab23
--- a/src/HOL/Complex.thy	Mon Dec 07 10:23:50 2015 +0100
+++ b/src/HOL/Complex.thy	Mon Dec 07 10:38:04 2015 +0100
@@ -11,8 +11,8 @@
 begin
 
 text \<open>
-We use the @{text codatatype} command to define the type of complex numbers. This allows us to use
-@{text primcorec} to define complex functions by defining their real and imaginary result
+We use the \<open>codatatype\<close> command to define the type of complex numbers. This allows us to use
+\<open>primcorec\<close> to define complex functions by defining their real and imaginary result
 separately.
 \<close>