# HG changeset patch # User desharna # Date 1738573499 -3600 # Node ID 361fbb3e21c8323a1207492cf98609a4aea21fa0 # Parent 8fd693bb01c5ed1c4f7ce27469cbcfb2e189f449 added lemma strict_partial_order_wfp_on_finite_set diff -r 8fd693bb01c5 -r 361fbb3e21c8 NEWS --- a/NEWS Sun Feb 02 21:53:08 2025 +0100 +++ b/NEWS Mon Feb 03 10:04:59 2025 +0100 @@ -302,6 +302,7 @@ wfP_wf_eq ~> wfp_wf_eq wf_acc_iff ~> wf_iff_acc - Added lemmas. + strict_partial_order_wfp_on_finite_set wf_on_antimono_stronger wfp_on_antimono_stronger diff -r 8fd693bb01c5 -r 361fbb3e21c8 src/HOL/Wellfounded.thy --- a/src/HOL/Wellfounded.thy Sun Feb 02 21:53:08 2025 +0100 +++ b/src/HOL/Wellfounded.thy Mon Feb 03 10:04:59 2025 +0100 @@ -307,6 +307,33 @@ lemmas wfp_eq_minimal = wf_eq_minimal [to_pred] +subsubsection \Finite characterization of well-foundedness\ + +lemma strict_partial_order_wfp_on_finite_set: + assumes "transp_on \ R" and "asymp_on \ R" and "finite \" + shows "wfp_on \ R" + unfolding Wellfounded.wfp_on_iff_ex_minimal +proof (intro allI impI) + fix \ + assume "\ \ \" and "\ \ {}" + + have "finite \" + using finite_subset[OF \\ \ \\ \finite \\] . + + moreover have "asymp_on \ R" + using asymp_on_subset[OF \asymp_on \ R\ \\ \ \\] . + + moreover have "transp_on \ R" + using transp_on_subset[OF \transp_on \ R\ \\ \ \\] . + + ultimately have "\m\\. \x\\. x \ m \ \ R x m" + using \\ \ {}\ Finite_Set.bex_min_element[of \ R] by iprover + + thus "\z\\. \y. R y z \ y \ \" + using asymp_onD[OF \asymp_on \ R\] by fast +qed + + subsubsection \Antimonotonicity\