Documentation

Mathlib.Data.Set.BoolIndicator

Indicator function valued in bool #

See also Set.indicator and Set.piecewise.

noncomputable def Set.boolIndicator {α : Type u_1} (s : Set α) (x : α) :

boolIndicator maps x to true if x ∈ s, else to false

Equations
Instances For
    theorem Set.mem_iff_boolIndicator {α : Type u_1} (s : Set α) (x : α) :
    x s s.boolIndicator x = true
    theorem Set.not_mem_iff_boolIndicator {α : Type u_1} (s : Set α) (x : α) :
    xs s.boolIndicator x = false
    theorem Set.preimage_boolIndicator_true {α : Type u_1} (s : Set α) :
    s.boolIndicator ⁻¹' {true} = s
    theorem Set.preimage_boolIndicator_false {α : Type u_1} (s : Set α) :
    s.boolIndicator ⁻¹' {false} = s
    theorem Set.preimage_boolIndicator_eq_union {α : Type u_1} (s : Set α) (t : Set Bool) :
    s.boolIndicator ⁻¹' t = (if true t then s else ) if false t then s else
    theorem Set.preimage_boolIndicator {α : Type u_1} (s : Set α) (t : Set Bool) :
    s.boolIndicator ⁻¹' t = Set.univ s.boolIndicator ⁻¹' t = s s.boolIndicator ⁻¹' t = s s.boolIndicator ⁻¹' t =