Skip to content

Commit

Permalink
Feat: add Sigma.map_mk (#1905)
Browse files Browse the repository at this point in the history
`simp [Sigma.map_mk]` has the same effect in Lean 4 as `simp [sigma.map]` has in Lean 3. OTOH, `simp [Sigma.map]` unfolds non-applied `Sigma.map`s too.
  • Loading branch information
urkud committed Jan 31, 2023
1 parent ebfc908 commit 4809cc9
Showing 1 changed file with 2 additions and 0 deletions.
2 changes: 2 additions & 0 deletions Mathlib/Data/Sigma/Basic.lean
Expand Up @@ -102,6 +102,8 @@ def map (f₁ : α₁ → α₂) (f₂ : ∀ a, β₁ a → β₂ (f₁ a)) (x :
⟨f₁ x.1, f₂ x.1 x.2
#align sigma.map Sigma.map

lemma map_mk (f₁ : α₁ → α₂) (f₂ : ∀ a, β₁ a → β₂ (f₁ a)) (x : α₁) (y : β₁ x) :
map f₁ f₂ ⟨x, y⟩ = ⟨f₁ x, f₂ x y⟩ := rfl
end Sigma

theorem sigma_mk_injective {i : α} : Function.Injective (@Sigma.mk α β i)
Expand Down

0 comments on commit 4809cc9

Please sign in to comment.