diff -r d33fc5228aae -r 44a3e883ccda src/HOL/Relation.thy --- a/src/HOL/Relation.thy Mon Dec 19 15:33:13 2022 +0100 +++ b/src/HOL/Relation.thy Tue Dec 20 08:41:01 2022 +0100 @@ -663,8 +663,13 @@ lemma transp_INF: "\x\S. transp (r x) \ transp (\(r ` S))" by (fact trans_INTER [to_pred]) - -lemma trans_join [code]: "trans r \ (\(x, y1) \ r. \(y2, z) \ r. y1 = y2 \ (x, z) \ r)" + +lemma trans_on_join [code]: + "trans_on A r \ (\(x, y1) \ r. x \ A \ y1 \ A \ + (\(y2, z) \ r. y1 = y2 \ z \ A \ (x, z) \ r))" + by (auto simp: trans_on_def) + +lemma trans_join: "trans r \ (\(x, y1) \ r. \(y2, z) \ r. y1 = y2 \ (x, z) \ r)" by (auto simp add: trans_def) lemma transp_trans: "transp r \ trans {(x, y). r x y}"