moved left_unique_conversep[simp] and right_unique_conversep[simp] to HOL.Relation
authordesharna
Sun, 16 Mar 2025 09:11:17 +0100
changeset 82286 4042628fffa5
parent 82285 d804c8e78ed3
child 82287 6ace531790b4
child 82291 3cb05c9ce8c4
moved left_unique_conversep[simp] and right_unique_conversep[simp] to HOL.Relation
src/HOL/Relation.thy
src/HOL/Transfer.thy
--- a/src/HOL/Relation.thy	Sat Mar 15 22:42:29 2025 +0100
+++ b/src/HOL/Relation.thy	Sun Mar 16 09:11:17 2025 +0100
@@ -1283,6 +1283,12 @@
 lemma totalp_on_converse [simp]: "totalp_on A R\<inverse>\<inverse> = totalp_on A R"
   by (rule total_on_converse[to_pred])
 
+lemma left_unique_conversep[simp]: "left_unique A\<inverse>\<inverse> \<longleftrightarrow> right_unique A"
+  by (auto simp add: left_unique_def right_unique_def)
+
+lemma right_unique_conversep[simp]: "right_unique A\<inverse>\<inverse> \<longleftrightarrow> left_unique A"
+  by (auto simp add: left_unique_def right_unique_def)
+
 lemma conversep_noteq [simp]: "(\<noteq>)\<inverse>\<inverse> = (\<noteq>)"
   by (auto simp add: fun_eq_iff)
 
--- a/src/HOL/Transfer.thy	Sat Mar 15 22:42:29 2025 +0100
+++ b/src/HOL/Transfer.thy	Sun Mar 16 09:11:17 2025 +0100
@@ -182,11 +182,6 @@
   unfolding bi_unique_def rel_fun_def by auto
 
 lemma [simp]:
-  shows left_unique_conversep: "left_unique A\<inverse>\<inverse> \<longleftrightarrow> right_unique A"
-    and right_unique_conversep: "right_unique A\<inverse>\<inverse> \<longleftrightarrow> left_unique A"
-  by(auto simp add: left_unique_def right_unique_def)
-
-lemma [simp]:
   shows left_total_conversep: "left_total A\<inverse>\<inverse> \<longleftrightarrow> right_total A"
     and right_total_conversep: "right_total A\<inverse>\<inverse> \<longleftrightarrow> left_total A"
   by(simp_all add: left_total_def right_total_def)