We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
1 parent cf1c5c2 commit bacc8b0Copy full SHA for bacc8b0
Mathlib/Data/Set/Subset.lean
@@ -112,8 +112,10 @@ lemma image_val_union_self_left_eq : ↑D ∪ A = A :=
112
union_eq_right.2 image_val_subset
113
114
@[simp]
115
-lemma cou_inter_self_right_eq_coe : A ∩ ↑D = ↑D :=
+lemma image_val_inter_self_right_eq_coe : A ∩ ↑D = ↑D :=
116
inter_eq_right.2 image_val_subset
117
+@[deprecated (since := "2024-10-25")]
118
+alias cou_inter_self_right_eq_coe := image_val_inter_self_right_eq_coe
119
120
121
lemma image_val_inter_self_left_eq_coe : ↑D ∩ A = ↑D :=
0 commit comments