Piecewise functions #
This file contains basic results on piecewise defined functions.
theorem
Set.piecewise_singleton
{α : Type u_1}
{β : Type u_2}
(x : α)
[(y : α) → Decidable (y ∈ {x})]
[DecidableEq α]
(f g : α → β)
:
@[deprecated Set.piecewise_mono (since := "2024-10-06")]
theorem
Set.piecewise_le_piecewise
{α : Type u_1}
{δ : α → Type u_8}
[(i : α) → Preorder (δ i)]
{s : Set α}
[(j : α) → Decidable (j ∈ s)]
{f₁ f₂ g₁ g₂ : (i : α) → δ i}
(h₁ : ∀ i ∈ s, f₁ i ≤ g₁ i)
(h₂ : ∀ i ∉ s, f₂ i ≤ g₂ i)
:
Alias of Set.piecewise_mono
.