src/ZF/Induct/Binary_Trees.thy
changeset 67443 3abf6a722518
parent 65449 c82e63b11b8b
child 69593 3dda49e08b9d
--- a/src/ZF/Induct/Binary_Trees.thy	Tue Jan 16 09:12:16 2018 +0100
+++ b/src/ZF/Induct/Binary_Trees.thy	Tue Jan 16 09:30:00 2018 +0100
@@ -21,11 +21,11 @@
   by (induct arbitrary: x r set: bt) auto
 
 lemma Br_iff: "Br(a, l, r) = Br(a', l', r') \<longleftrightarrow> a = a' & l = l' & r = r'"
-  \<comment> "Proving a freeness theorem."
+  \<comment> \<open>Proving a freeness theorem.\<close>
   by (fast elim!: bt.free_elims)
 
 inductive_cases BrE: "Br(a, l, r) \<in> bt(A)"
-  \<comment> "An elimination rule, for type-checking."
+  \<comment> \<open>An elimination rule, for type-checking.\<close>
 
 text \<open>
   \medskip Lemmas to justify using @{term bt} in other recursive type