src/ZF/Induct/Ntree.thy
changeset 69593 3dda49e08b9d
parent 65449 c82e63b11b8b
child 76213 e44d86131648
--- a/src/ZF/Induct/Ntree.thy	Fri Jan 04 21:49:06 2019 +0100
+++ b/src/ZF/Induct/Ntree.thy	Fri Jan 04 23:22:53 2019 +0100
@@ -69,7 +69,7 @@
     and step: "!!x n h. [| x \<in> A;  n \<in> nat;  h \<in> n -> ntree(A);  f O h = g O h |] ==>
       f ` Branch(x,h) = g ` Branch(x,h)"
   shows "f`t=g`t"
-  \<comment> \<open>Induction on @{term "ntree(A)"} to prove an equation\<close>
+  \<comment> \<open>Induction on \<^term>\<open>ntree(A)\<close> to prove an equation\<close>
   using t
   apply induct
   apply (assumption | rule step)+