Skip to content

Commit

Permalink
rephrase
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em committed Jun 24, 2024
1 parent ec3b4c9 commit a0d6d20
Showing 1 changed file with 2 additions and 3 deletions.
5 changes: 2 additions & 3 deletions Mathlib/Data/Prod/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -61,9 +61,8 @@ theorem map_mk (f : α → γ) (g : β → δ) (a : α) (b : β) : map f g (a, b
rfl
#align prod.map_mk Prod.map_mk

-- I'm skeptical about having this as a `simp` lemma, despite it having been in the past
-- as it destructures the pair. See `map_apply`, `map_fst`, and `map_snd` for slightly weaker
-- lemmas in the `simp` set.
-- This was previously a `simp` lemma, but no longer is on the basis that it destructures the pair.
-- See `map_apply`, `map_fst`, and `map_snd` for slightly weaker lemmas in the `simp` set.
theorem map_apply' (f : α → γ) (g : β → δ) (p : α × β) : map f g p = (f p.1, g p.2) :=
rfl

Expand Down

0 comments on commit a0d6d20

Please sign in to comment.