src/HOL/Data_Structures/Tree_Set.thy
changeset 61231 cc6969542f8d
parent 61229 0b9c45c4af29
child 61428 5e1938107371
--- a/src/HOL/Data_Structures/Tree_Set.thy	Tue Sep 22 17:13:13 2015 +0200
+++ b/src/HOL/Data_Structures/Tree_Set.thy	Wed Sep 23 09:14:22 2015 +0200
@@ -43,7 +43,7 @@
 
 lemma inorder_insert:
   "sorted(inorder t) \<Longrightarrow> inorder(insert x t) = ins_list x (inorder t)"
-by(induction t) (auto simp: ins_simps)
+by(induction t) (auto simp: ins_list_simps)
 
 
 lemma del_minD:
@@ -54,7 +54,7 @@
 
 lemma inorder_delete:
   "sorted(inorder t) \<Longrightarrow> inorder(delete x t) = del_list x (inorder t)"
-by(induction t) (auto simp: del_simps del_minD split: prod.splits)
+by(induction t) (auto simp: del_list_simps del_minD split: prod.splits)
 
 
 interpretation Set_by_Ordered