# HG changeset patch # User nipkow # Date 1596903609 -7200 # Node ID 2dcb6523f6af0441adffbc7e731cf7a4dcf448f2 # Parent 42f931a6885607993ffc7e00e30da658d0089a1a tuned diff -r 42f931a68856 -r 2dcb6523f6af src/HOL/Data_Structures/Tree23_of_List.thy --- 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 \Completeness:\