src/HOL/Computational_Algebra/Formal_Power_Series.thy
changeset 69597 ff784d5a5bfb
parent 69325 4b6ddc5989fc
child 69791 195aeee8b30a
--- a/src/HOL/Computational_Algebra/Formal_Power_Series.thy	Sat Jan 05 17:00:43 2019 +0100
+++ b/src/HOL/Computational_Algebra/Formal_Power_Series.thy	Sat Jan 05 17:24:33 2019 +0100
@@ -4533,7 +4533,7 @@
   finally show ?thesis by simp
 qed
 
-text \<open>Connection to @{const "fps_exp"} over the complex numbers --- Euler and de Moivre.\<close>
+text \<open>Connection to \<^const>\<open>fps_exp\<close> over the complex numbers --- Euler and de Moivre.\<close>
 
 lemma fps_exp_ii_sin_cos: "fps_exp (\<i> * c) = fps_cos c + fps_const \<i> * fps_sin c"
   (is "?l = ?r")