src/HOL/Library/Ramsey.thy
changeset 58622 aa99568f56de
parent 54580 7b9336176a1c
child 58881 b9556a055632
equal deleted inserted replaced
58621:7a2c567061b3 58622:aa99568f56de
   336 
   336 
   337 subsection {* Disjunctive Well-Foundedness *}
   337 subsection {* Disjunctive Well-Foundedness *}
   338 
   338 
   339 text {*
   339 text {*
   340   An application of Ramsey's theorem to program termination. See
   340   An application of Ramsey's theorem to program termination. See
   341   \cite{Podelski-Rybalchenko}.
   341   @{cite "Podelski-Rybalchenko"}.
   342 *}
   342 *}
   343 
   343 
   344 definition disj_wf :: "('a * 'a)set => bool"
   344 definition disj_wf :: "('a * 'a)set => bool"
   345   where "disj_wf r = (\<exists>T. \<exists>n::nat. (\<forall>i<n. wf(T i)) & r = (\<Union>i<n. T i))"
   345   where "disj_wf r = (\<exists>T. \<exists>n::nat. (\<forall>i<n. wf(T i)) & r = (\<Union>i<n. T i))"
   346 
   346