Skip to content

Commit

Permalink
chore: remove reducible from Function.Surjective (#5063)
Browse files Browse the repository at this point in the history
The @[reducible] attribute on `Function.Surjective` is apparently not needed, and currently prevents `@[simp]` lemmas with `Function.Surjective` side conditions from firing, see [zulip discussion](https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/simp.20lemmas.20with.20side.20conditions).



Co-authored-by: Scott Morrison <[email protected]>
  • Loading branch information
kim-em and Scott Morrison committed Jun 15, 2023
1 parent dd52d5f commit 28ad0a6
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion Mathlib/Init/Function.lean
Original file line number Diff line number Diff line change
Expand Up @@ -68,7 +68,7 @@ fun _ _ h ↦ hf (hg h)

/-- A function `f : α → β` is called surjective if every `b : β` is equal to `f a`
for some `a : α`. -/
@[reducible] def Surjective (f : α → β) : Prop := ∀ b, ∃ a, f a = b
def Surjective (f : α → β) : Prop := ∀ b, ∃ a, f a = b

theorem Surjective.comp {g : β → φ} {f : α → β} (hg : Surjective g) (hf : Surjective f) :
Surjective (g ∘ f) :=
Expand Down

0 comments on commit 28ad0a6

Please sign in to comment.