diff -r 785c0f6b8184 -r 20c1d3a14143 RTree.thy --- a/RTree.thy Wed Aug 24 16:13:20 2016 +0200 +++ b/RTree.thy Sun Oct 02 14:32:05 2016 +0100 @@ -77,6 +77,27 @@ definition "ancestors r x = {y. (x, y) \ r^+}" +(* tmp *) +definition + "nancestors r x \ ancestors r x \ {x}" + +lemma nancestors_def2: + "nancestors r x \ {y. (x, y) \ r\<^sup>*}" +unfolding nancestors_def +apply(auto) +by (smt Collect_cong ancestors_def insert_compr mem_Collect_eq rtrancl_eq_or_trancl) + +lemma nancestors2: + "y \ ancestors r x \ y \ nancestors r x" +apply(auto simp add: nancestors_def) +done + +lemma nancestors3: + "\y \ nancestors r x; x \ y\ \ y \ ancestors r x" +apply(auto simp add: nancestors_def) +done +(* end tmp *) + definition "root r x = (ancestors r x = {})" lemma root_indep: