diff -r 02719bd7b4e6 -r a4fa039a6a60 src/HOL/Relation.thy --- a/src/HOL/Relation.thy Sat Jun 04 18:32:30 2022 +0200 +++ b/src/HOL/Relation.thy Sat Jun 04 19:11:52 2022 +0200 @@ -528,6 +528,9 @@ abbreviation totalp where "totalp \ totalp_on UNIV" +lemma totalp_on_refl_on_eq[pred_set_conv]: "totalp_on A (\x y. (x, y) \ r) \ total_on A r" + by (simp add: totalp_on_def total_on_def) + lemma totalp_onI: "(\x y. x \ A \ y \ A \ x \ y \ R x y \ R y x) \ totalp_on A R" by (simp add: totalp_on_def)