src/HOL/Power.thy
changeset 69593 3dda49e08b9d
parent 68611 4bc4b5c0ccfc
child 69700 7a92cbec7030
--- a/src/HOL/Power.thy	Fri Jan 04 21:49:06 2019 +0100
+++ b/src/HOL/Power.thy	Fri Jan 04 23:22:53 2019 +0100
@@ -457,7 +457,7 @@
   by (force simp add: order_antisym power_le_imp_le_exp)
 
 text \<open>
-  Can relax the first premise to @{term "0<a"} in the case of the
+  Can relax the first premise to \<^term>\<open>0<a\<close> in the case of the
   natural numbers.
 \<close>
 lemma power_less_imp_less_exp: "1 < a \<Longrightarrow> a ^ m < a ^ n \<Longrightarrow> m < n"