Indicator function valued in bool #
See also Set.indicator
and Set.piecewise
.
boolIndicator
maps x
to true
if x ∈ s
, else to false
Instances For
theorem
Set.preimage_boolIndicator
{α : Type u_1}
(s : Set α)
(t : Set Bool)
:
s.boolIndicator ⁻¹' t = univ ∨ s.boolIndicator ⁻¹' t = s ∨ s.boolIndicator ⁻¹' t = sᶜ ∨ s.boolIndicator ⁻¹' t = ∅