src/HOL/Relation.thy
changeset 82270 4355a2afa7a3
parent 82248 e8c96013ea8a
child 82271 f7e08143eea2
--- a/src/HOL/Relation.thy	Thu Mar 13 16:00:48 2025 +0100
+++ b/src/HOL/Relation.thy	Fri Mar 14 18:02:16 2025 +0100
@@ -167,8 +167,10 @@
 
 text \<open>@{thm [source] reflp_def} is for backward compatibility.\<close>
 
-lemma reflp_refl_eq [pred_set_conv]: "reflp (\<lambda>x y. (x, y) \<in> r) \<longleftrightarrow> refl r"
-  by (simp add: refl_on_def reflp_def)
+lemma reflp_on_refl_on_eq[pred_set_conv]: "reflp_on A (\<lambda>a b. (a, b) \<in> r) \<longleftrightarrow> refl_on A r"
+  by (simp add: refl_on_def reflp_on_def)
+
+lemmas reflp_refl_eq = reflp_on_refl_on_eq[of UNIV]
 
 lemma refl_onI [intro?]: "(\<And>x. x \<in> A \<Longrightarrow> (x, x) \<in> r) \<Longrightarrow> refl_on A r"
   unfolding refl_on_def by (iprover intro!: ballI)