diff -r 458b4e3720ab -r 27f3c10b0b50 src/ZF/Induct/Binary_Trees.thy --- a/src/ZF/Induct/Binary_Trees.thy Mon Dec 07 10:19:30 2015 +0100 +++ b/src/ZF/Induct/Binary_Trees.thy Mon Dec 07 10:23:50 2015 +0100 @@ -21,11 +21,11 @@ by (induct arbitrary: x r set: bt) auto lemma Br_iff: "Br(a, l, r) = Br(a', l', r') \ a = a' & l = l' & r = r'" - -- "Proving a freeness theorem." + \ "Proving a freeness theorem." by (fast elim!: bt.free_elims) inductive_cases BrE: "Br(a, l, r) \ bt(A)" - -- "An elimination rule, for type-checking." + \ "An elimination rule, for type-checking." text \ \medskip Lemmas to justify using @{term bt} in other recursive type @@ -58,7 +58,7 @@ !!x y z r s. [| x \ A; y \ bt(A); z \ bt(A); r \ C(y); s \ C(z) |] ==> h(x, y, z, r, s) \ C(Br(x, y, z)) |] ==> bt_rec(c, h, t) \ C(t)" - -- \Type checking for recursor -- example only; not really needed.\ + \ \Type checking for recursor -- example only; not really needed.\ apply (induct_tac t) apply simp_all done