src/HOL/Data_Structures/Tree23_of_List.thy
changeset 72122 2dcb6523f6af
parent 72121 42f931a68856
child 72543 66d09b9da6a2
--- a/src/HOL/Data_Structures/Tree23_of_List.thy	Sat Aug 08 18:04:08 2020 +0200
+++ b/src/HOL/Data_Structures/Tree23_of_List.thy	Sat Aug 08 18:20:09 2020 +0200
@@ -87,7 +87,7 @@
 lemma inorder2_leaves: "inorder2(leaves as) = as"
 by(induction as) auto
 
-lemma "inorder(tree23_of_list as) = as"
+lemma inorder: "inorder(tree23_of_list as) = as"
 by(simp add: tree23_of_list_def inorder_join_all inorder2_leaves)
 
 subsubsection \<open>Completeness:\<close>