src/HOL/Complex.thy
changeset 65579 52eafedaf196
parent 65578 e4997c181cce
child 65583 8d53b3bebab4
--- a/src/HOL/Complex.thy	Tue Apr 25 16:39:54 2017 +0100
+++ b/src/HOL/Complex.thy	Tue Apr 25 17:10:17 2017 +0100
@@ -138,7 +138,7 @@
 end
 
 
-subsection \<open>Numerals, Arithmetic, and Embedding from \<real>\<close>
+subsection \<open>Numerals, Arithmetic, and Embedding from R\<close>
 
 abbreviation complex_of_real :: "real \<Rightarrow> complex"
   where "complex_of_real \<equiv> of_real"