src/HOL/Accessible_Part.thy
changeset 21404 eb85850d3eb7
parent 19669 95ac857276e1
child 22262 96ba62dff413
equal deleted inserted replaced
21403:dd58f13a8eb4 21404:eb85850d3eb7
    22 inductive "acc r"
    22 inductive "acc r"
    23   intros
    23   intros
    24     accI: "(!!y. (y, x) \<in> r ==> y \<in> acc r) ==> x \<in> acc r"
    24     accI: "(!!y. (y, x) \<in> r ==> y \<in> acc r) ==> x \<in> acc r"
    25 
    25 
    26 abbreviation
    26 abbreviation
    27   termi :: "('a \<times> 'a) set => 'a set"
    27   termi :: "('a \<times> 'a) set => 'a set" where
    28   "termi r == acc (r\<inverse>)"
    28   "termi r == acc (r\<inverse>)"
    29 
    29 
    30 
    30 
    31 subsection {* Induction rules *}
    31 subsection {* Induction rules *}
    32 
    32