merged
authordesharna
Sun, 04 Dec 2022 18:49:58 +0100
changeset 76555 e28aed61a4b1
parent 76553 120f79cdb492 (current diff)
parent 76554 a7d9e34c85e6 (diff)
child 76556 c7f3e94fce7b
merged
--- a/src/HOL/Relation.thy	Sun Dec 04 14:24:42 2022 +0100
+++ b/src/HOL/Relation.thy	Sun Dec 04 18:49:58 2022 +0100
@@ -90,10 +90,10 @@
 lemma bot_empty_eq2 [pred_set_conv]: "\<bottom> = (\<lambda>x y. (x, y) \<in> {})"
   by (auto simp add: fun_eq_iff)
 
-lemma top_empty_eq [pred_set_conv]: "\<top> = (\<lambda>x. x \<in> UNIV)"
+lemma top_empty_eq: "\<top> = (\<lambda>x. x \<in> UNIV)"
   by (auto simp add: fun_eq_iff)
 
-lemma top_empty_eq2 [pred_set_conv]: "\<top> = (\<lambda>x y. (x, y) \<in> UNIV)"
+lemma top_empty_eq2: "\<top> = (\<lambda>x y. (x, y) \<in> UNIV)"
   by (auto simp add: fun_eq_iff)
 
 lemma inf_Int_eq [pred_set_conv]: "(\<lambda>x. x \<in> R) \<sqinter> (\<lambda>x. x \<in> S) = (\<lambda>x. x \<in> R \<inter> S)"