src/HOL/Data_Structures/Isin2.thy
changeset 67967 5a4280946a25
parent 67965 aaa31cd0caef
child 68413 b56ed5010e69
--- a/src/HOL/Data_Structures/Isin2.thy	Sun Apr 08 12:14:00 2018 +0200
+++ b/src/HOL/Data_Structures/Isin2.thy	Sun Apr 08 12:31:08 2018 +0200
@@ -17,7 +17,10 @@
      EQ \<Rightarrow> True |
      GT \<Rightarrow> isin r x)"
 
-lemma isin_set: "sorted(inorder t) \<Longrightarrow> isin t x = (x \<in> set(inorder t))"
+lemma isin_set_inorder: "sorted(inorder t) \<Longrightarrow> isin t x = (x \<in> set(inorder t))"
 by (induction t) (auto simp: isin_simps)
 
+lemma isin_set_tree: "bst t \<Longrightarrow> isin t x \<longleftrightarrow> x \<in> set_tree t"
+by(induction t) auto
+
 end