N-ary images of sets #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
This file defines finset.image₂
, the binary image of finsets. This is the finset version of
set.image2
. This is mostly useful to define pointwise operations.
Notes #
This file is very similar to the n-ary section of data.set.basic
, to order.filter.n_ary
and to
data.option.n_ary
. Please keep them in sync.
We do not define finset.image₃
as its only purpose would be to prove properties of finset.image₂
and set.image2
already fulfills this task.
The image of a binary function f : α → β → γ
as a function set α → set β → set γ
.
Mathematically this should be thought of as the image of the corresponding function α × β → γ
.
Instances for ↥set.image2
image2 is monotone with respect to ⊆
.
A common special case of image2_congr
The image of a ternary function f : α → β → γ → δ
as a function
set α → set β → set γ → set δ
. Mathematically this should be thought of as the image of the
corresponding function α × β × γ → δ
.
Symmetric statement to set.image2_image_left_comm
.
Symmetric statement to set.image_image2_right_comm
.
Symmetric statement to set.image_image2_distrib_left
.
Symmetric statement to set.image_image2_distrib_right
.
The other direction does not hold because of the s
-s
cross terms on the RHS.
The other direction does not hold because of the u
-u
cross terms on the RHS.
Symmetric statement to set.image2_image_left_anticomm
.
Symmetric statement to set.image_image2_right_anticomm
.
Symmetric statement to set.image_image2_antidistrib_left
.
Symmetric statement to set.image_image2_antidistrib_right
.
If a
is a left identity for f : α → β → β
, then {a}
is a left identity for
set.image2 f
.
If b
is a right identity for f : α → β → α
, then {b}
is a right identity for
set.image2 f
.