diff -r f7c5a010115a -r a01ea04aa58f src/HOL/Transfer.thy --- a/src/HOL/Transfer.thy Sat Mar 15 20:27:25 2025 +0100 +++ b/src/HOL/Transfer.thy Sat Mar 15 20:33:19 2025 +0100 @@ -106,6 +106,8 @@ subsection \Predicates on relations, i.e. ``class constraints''\ +text \See also \<^const>\Relation.left_unique\ and \<^const>\Relation.right_unique\.\ + definition left_total :: "('a \ 'b \ bool) \ bool" where "left_total R \ (\x. \y. R x y)" @@ -120,9 +122,6 @@ (\x y z. R x y \ R x z \ y = z) \ (\x y z. R x z \ R y z \ x = y)" -lemma left_unique_iff: "left_unique R \ (\z. \\<^sub>\\<^sub>1x. R x z)" - unfolding Uniq_def left_unique_def by force - lemma left_totalI: "(\x. \y. R x y) \ left_total R" unfolding left_total_def by blast @@ -141,9 +140,6 @@ lemma bi_unique_iff: "bi_unique R \ (\z. \\<^sub>\\<^sub>1x. R x z) \ (\z. \\<^sub>\\<^sub>1x. R z x)" unfolding Uniq_def bi_unique_def by force -lemma right_unique_iff: "right_unique R \ (\z. \\<^sub>\\<^sub>1x. R z x)" - unfolding Uniq_def right_unique_def by force - lemma right_totalI: "(\y. \x. A x y) \ right_total A" by(simp add: right_total_def)