Skip to content

Commit 93ca565

Browse files
committed
fix Sigma.eta
1 parent b5a509b commit 93ca565

File tree

1 file changed

+4
-2
lines changed

1 file changed

+4
-2
lines changed

src/Init/Core.lean

Lines changed: 4 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -1481,9 +1481,11 @@ def Prod.map {α₁ : Type u₁} {α₂ : Type u₂} {β₁ : Type v₁} {β₂
14811481
theorem Exists.of_psigma_prop {α : Sort u} {p : α → Prop} : (PSigma (fun x => p x)) → Exists (fun x => p x)
14821482
| ⟨x, hx⟩ => ⟨x, hx⟩
14831483

1484-
protected theorem Sigma.eta {α : Type u} {β : α → Type v} {x : Sigma β} : Sigma.mk x.1 x.2 = x := rfl
1484+
@[simp]
1485+
protected theorem Sigma.eta {α : Type u} {β : α → Type v} (x : Sigma β) : Sigma.mk x.1 x.2 = x := rfl
14851486

1486-
protected theorem PSigma.eta {α : Sort u} {β : α → Sort v} {x : PSigma β} : PSigma.mk x.1 x.2 = x := rfl
1487+
@[simp]
1488+
protected theorem PSigma.eta {α : Sort u} {β : α → Sort v} (x : PSigma β) : PSigma.mk x.1 x.2 = x := rfl
14871489

14881490
protected theorem PSigma.mk_congr {α : Sort u} {β : α → Sort v} {a₁ a₂ : α} {b₁ : β a₁} {b₂ : β a₂}
14891491
(h₁ : a₁ = a₂) (h₂ : Eq.ndrec b₁ h₁ = b₂) : PSigma.mk a₁ b₁ = PSigma.mk a₂ b₂ := by

0 commit comments

Comments
 (0)