Skip to content

Commit

Permalink
chore: remove porting notes involving the ematch attribute (#11037)
Browse files Browse the repository at this point in the history
`ematch` is not coming back (and was already completely unused for years in Lean 3).
  • Loading branch information
grunweg committed Feb 28, 2024
1 parent 30f0627 commit 1896df5
Show file tree
Hide file tree
Showing 2 changed files with 0 additions and 15 deletions.
2 changes: 0 additions & 2 deletions Mathlib/Algebra/GroupWithZero/Power.lean
Expand Up @@ -56,8 +56,6 @@ open Int

variable {G₀ : Type*} [GroupWithZero G₀]

-- Porting note: removed `attribute [local ematch] le_of_lt`

theorem zero_zpow : ∀ z : ℤ, z ≠ 0 → (0 : G₀) ^ z = 0
| (n : ℕ), h => by
rw [zpow_coe_nat, zero_pow]
Expand Down
13 changes: 0 additions & 13 deletions Mathlib/Order/CompleteLattice.lean
Expand Up @@ -73,7 +73,6 @@ section

variable [CompleteSemilatticeSup α] {s t : Set α} {a b : α}

-- --@[ematch] Porting note: attribute removed
theorem le_sSup : a ∈ s → a ≤ sSup s :=
CompleteSemilatticeSup.le_sSup s a
#align le_Sup le_sSup
Expand Down Expand Up @@ -144,7 +143,6 @@ section

variable [CompleteSemilatticeInf α] {s t : Set α} {a b : α}

-- --@[ematch] Porting note: attribute removed
theorem sInf_le : a ∈ s → sInf s ≤ a :=
CompleteSemilatticeInf.sInf_le s a
#align Inf_le sInf_le
Expand Down Expand Up @@ -707,8 +705,6 @@ section

variable [CompleteLattice α] {f g s t : ι → α} {a b : α}

-- TODO: this declaration gives error when starting smt state
----@[ematch] Porting note: attribute removed
theorem le_iSup (f : ι → α) (i : ι) : f i ≤ iSup f :=
le_sSup ⟨i, rfl⟩
#align le_supr le_iSup
Expand All @@ -717,21 +713,14 @@ theorem iInf_le (f : ι → α) (i : ι) : iInf f ≤ f i :=
sInf_le ⟨i, rfl⟩
#align infi_le iInf_le

-- --@[ematch] Porting note: attribute removed
theorem le_iSup' (f : ι → α) (i : ι) : f i ≤ iSup f :=
le_sSup ⟨i, rfl⟩
#align le_supr' le_iSup'

----@[ematch] Porting note: attribute removed
theorem iInf_le' (f : ι → α) (i : ι) : iInf f ≤ f i :=
sInf_le ⟨i, rfl⟩
#align infi_le' iInf_le'

/- TODO: this version would be more powerful, but, alas, the pattern matcher
doesn't accept it.
--@[ematch] lemma le_iSup' (f : ι → α) (i : ι) : (: f i :) ≤ (: iSup f :) :=
le_sSup ⟨i, rfl⟩
-/
theorem isLUB_iSup : IsLUB (range f) (⨆ j, f j) :=
isLUB_sSup _
#align is_lub_supr isLUB_iSup
Expand Down Expand Up @@ -1154,8 +1143,6 @@ theorem iInf_iInf_eq_right {b : β} {f : ∀ x : β, b = x → α} : ⨅ x, ⨅
@iSup_iSup_eq_right αᵒᵈ _ _ _ _
#align infi_infi_eq_right iInf_iInf_eq_right

-- attribute [ematch] le_refl Porting note: removed attribute

theorem iSup_subtype {p : ι → Prop} {f : Subtype p → α} : iSup f = ⨆ (i) (h : p i), f ⟨i, h⟩ :=
le_antisymm (iSup_le fun ⟨i, h⟩ => @le_iSup₂ _ _ p _ (fun i h => f ⟨i, h⟩) i h)
(iSup₂_le fun _ _ => le_iSup _ _)
Expand Down

0 comments on commit 1896df5

Please sign in to comment.