src/HOL/Transfer.thy
changeset 82274 c61367ada9bb
parent 81100 6ae3d0b2b8ad
child 82275 c17902fcf5e7
--- a/src/HOL/Transfer.thy	Fri Mar 14 18:13:56 2025 +0100
+++ b/src/HOL/Transfer.thy	Sat Mar 15 09:17:46 2025 +0100
@@ -126,6 +126,9 @@
     (\<forall>x y z. R x y \<longrightarrow> R x z \<longrightarrow> y = z) \<and>
     (\<forall>x y z. R x z \<longrightarrow> R y z \<longrightarrow> x = y)"
 
+lemma single_valuedp_eq_right_unique: "single_valuedp = right_unique"
+  by (rule ext) (simp add: single_valuedp_def right_unique_def)
+
 lemma left_unique_iff: "left_unique R \<longleftrightarrow> (\<forall>z. \<exists>\<^sub>\<le>\<^sub>1x. R x z)"
   unfolding Uniq_def left_unique_def by force