Skip to content

Commit

Permalink
more unused variables
Browse files Browse the repository at this point in the history
  • Loading branch information
adomani committed Sep 29, 2024
1 parent 85ec489 commit aa0f8ba
Showing 1 changed file with 2 additions and 5 deletions.
7 changes: 2 additions & 5 deletions Mathlib/Data/Set/Function.lean
Original file line number Diff line number Diff line change
Expand Up @@ -166,8 +166,7 @@ end restrict
/-! ### Equality on a set -/
section equality

variable {s s₁ s₂ : Set α} {t t₁ t₂ : Set β} {p : Set γ} {f f₁ f₂ f₃ : α → β} {g g₁ g₂ : β → γ}
{f' f₁' f₂' : β → α} {g' : γ → β} {a : α} {b : β}
variable {s s₁ s₂ : Set α} {f₁ f₂ f₃ : α → β} {g : β → γ} {a : α}

@[simp]
theorem eqOn_empty (f₁ f₂ : α → β) : EqOn f₁ f₂ ∅ := fun _ => False.elim
Expand Down Expand Up @@ -233,7 +232,7 @@ alias ⟨EqOn.comp_eq, _⟩ := eqOn_range

end equality

variable {s s₁ s₂ : Set α} {t t₁ t₂ : Set β} {p : Set γ} {f f₁ f₂ f₃ : α → β} {g g₁ g₂ : β → γ}
variable {s s₁ s₂ : Set α} {t t₁ t₂ : Set β} {p : Set γ} {f f₁ f₂ : α → β} {g g₁ g₂ : β → γ}
{f' f₁' f₂' : β → α} {g' : γ → β} {a : α} {b : β}

section MapsTo
Expand Down Expand Up @@ -450,8 +449,6 @@ theorem preimage_restrictPreimage {u : Set t} :
rw [← preimage_preimage (g := f) (f := Subtype.val), ← image_val_preimage_restrictPreimage,
preimage_image_eq _ Subtype.val_injective]

variable {U : ι → Set β}

lemma restrictPreimage_injective (hf : Injective f) : Injective (t.restrictPreimage f) :=
fun _ _ e => Subtype.coe_injective <| hf <| Subtype.mk.inj e

Expand Down

0 comments on commit aa0f8ba

Please sign in to comment.