src/HOL/Relation.thy
changeset 82272 a317d9e27a03
parent 82271 f7e08143eea2
child 82273 365917fc6e31
--- a/src/HOL/Relation.thy	Fri Mar 14 18:04:14 2025 +0100
+++ b/src/HOL/Relation.thy	Fri Mar 14 18:11:38 2025 +0100
@@ -589,9 +589,8 @@
   "antisymp \<bottom>"
   by (fact antisym_empty [to_pred])
     
-lemma antisymp_equality [simp]:
-  "antisymp HOL.eq"
-  by (auto intro: antisympI)
+lemma antisymp_on_equality[simp]: "antisymp_on A (=)"
+  by (auto intro: antisymp_onI)
 
 lemma antisym_singleton [simp]:
   "antisym {x}"
@@ -715,8 +714,8 @@
 lemma transp_trans: "transp r \<longleftrightarrow> trans {(x, y). r x y}"
   by (simp add: trans_def transp_def)
 
-lemma transp_equality [simp]: "transp (=)"
-  by (auto intro: transpI)
+lemma transp_on_equality[simp]: "transp_on A (=)"
+  by (auto intro: transp_onI)
 
 lemma trans_empty [simp]: "trans {}"
   by (blast intro: transI)