# HG changeset patch # User desharna # Date 1742890244 -3600 # Node ID 4238ebc9918d94c9500acb9504969a0c7afb8e11 # Parent 25019484aa6d60eb68e3cc3d795acf2c65268360 renamed lemmas diff -r 25019484aa6d -r 4238ebc9918d NEWS --- a/NEWS Tue Mar 25 09:41:01 2025 +0100 +++ b/NEWS Tue Mar 25 09:10:44 2025 +0100 @@ -99,6 +99,13 @@ transp_on_top[simp] * Theory "HOL.Wellfounded": + - Renamed lemmas. Minor INCOMPATIBILITY. + wf_on_antimono_stronger ~> wf_on_mono_stronger + wf_on_antimono_strong ~> wf_on_mono_strong + wf_on_antimono ~> wf_on_mono + wfp_on_antimono_stronger ~> wfp_on_mono_stronger + wfp_on_antimono_strong ~> wfp_on_mono_strong + wfp_on_antimono ~> wfp_on_mono - Removed lemmas. Minor INCOMPATIBILITY. wf_empty[iff] (use wf_on_bot instead) - Added lemmas. diff -r 25019484aa6d -r 4238ebc9918d src/HOL/Wellfounded.thy --- a/src/HOL/Wellfounded.thy Tue Mar 25 09:41:01 2025 +0100 +++ b/src/HOL/Wellfounded.thy Tue Mar 25 09:10:44 2025 +0100 @@ -337,7 +337,7 @@ subsubsection \Antimonotonicity\ -lemma wfp_on_antimono_stronger: +lemma wfp_on_mono_stronger: fixes A :: "'a set" and B :: "'b set" and f :: "'a \ 'b" and @@ -363,34 +363,34 @@ using \A' \ A\ mono by blast qed -lemma wf_on_antimono_stronger: +lemma wf_on_mono_stronger: assumes "wf_on B r" and "f ` A \ B" and "(\x y. x \ A \ y \ A \ (x, y) \ q \ (f x, f y) \ r)" shows "wf_on A q" - using assms wfp_on_antimono_stronger[to_set, of B r f A q] by blast + using assms wfp_on_mono_stronger[to_set, of B r f A q] by blast -lemma wf_on_antimono_strong: +lemma wf_on_mono_strong: assumes "wf_on B r" and "A \ B" and "(\x y. x \ A \ y \ A \ (x, y) \ q \ (x, y) \ r)" shows "wf_on A q" - using assms wf_on_antimono_stronger[of B r "\x. x" A q] by blast + using assms wf_on_mono_stronger[of B r "\x. x" A q] by blast -lemma wfp_on_antimono_strong: +lemma wfp_on_mono_strong: "wfp_on B R \ A \ B \ (\x y. x \ A \ y \ A \ Q x y \ R x y) \ wfp_on A Q" - using wf_on_antimono_strong[of B _ A, to_pred] . + using wf_on_mono_strong[of B _ A, to_pred] . -lemma wf_on_antimono: "A \ B \ q \ r \ wf_on B r \ wf_on A q" - using wf_on_antimono_strong[of B r A q] by auto +lemma wf_on_mono: "A \ B \ q \ r \ wf_on B r \ wf_on A q" + using wf_on_mono_strong[of B r A q] by auto -lemma wfp_on_antimono: "A \ B \ Q \ R \ wfp_on B R \ wfp_on A Q" - using wfp_on_antimono_strong[of B R A Q] by auto +lemma wfp_on_mono: "A \ B \ Q \ R \ wfp_on B R \ wfp_on A Q" + using wfp_on_mono_strong[of B R A Q] by auto lemma wf_on_subset: "wf_on B r \ A \ B \ wf_on A r" - using wf_on_antimono_strong . + using wf_on_mono_strong . lemma wfp_on_subset: "wfp_on B R \ A \ B \ wfp_on A R" - using wfp_on_antimono_strong . + using wfp_on_mono_strong . subsubsection \Equivalence between \<^const>\wfp_on\ and \<^const>\wfp\\ @@ -405,7 +405,7 @@ next assume ?RHS thus ?LHS - proof (rule wfp_on_antimono_strong) + proof (rule wfp_on_mono_strong) show "A \ UNIV" using subset_UNIV . next @@ -524,7 +524,7 @@ text \Well-foundedness of subsets\ lemma wf_subset: "wf r \ p \ r \ wf p" - using wf_on_antimono[OF subset_UNIV, unfolded le_bool_def] .. + using wf_on_mono[OF subset_UNIV, unfolded le_bool_def] .. lemmas wfp_subset = wf_subset [to_pred]