src/HOL/Data_Structures/Isin2.thy
changeset 67967 5a4280946a25
parent 67965 aaa31cd0caef
child 68413 b56ed5010e69
equal deleted inserted replaced
67966:f13796496e82 67967:5a4280946a25
    15   (case cmp x a of
    15   (case cmp x a of
    16      LT \<Rightarrow> isin l x |
    16      LT \<Rightarrow> isin l x |
    17      EQ \<Rightarrow> True |
    17      EQ \<Rightarrow> True |
    18      GT \<Rightarrow> isin r x)"
    18      GT \<Rightarrow> isin r x)"
    19 
    19 
    20 lemma isin_set: "sorted(inorder t) \<Longrightarrow> isin t x = (x \<in> set(inorder t))"
    20 lemma isin_set_inorder: "sorted(inorder t) \<Longrightarrow> isin t x = (x \<in> set(inorder t))"
    21 by (induction t) (auto simp: isin_simps)
    21 by (induction t) (auto simp: isin_simps)
    22 
    22 
       
    23 lemma isin_set_tree: "bst t \<Longrightarrow> isin t x \<longleftrightarrow> x \<in> set_tree t"
       
    24 by(induction t) auto
       
    25 
    23 end
    26 end