Skip to content

Commit

Permalink
chore: update Std (#12210)
Browse files Browse the repository at this point in the history
Co-authored-by: Scott Morrison <scott.morrison@gmail.com>
  • Loading branch information
semorrison and semorrison committed Apr 18, 2024
1 parent a643996 commit dc34930
Show file tree
Hide file tree
Showing 5 changed files with 5 additions and 6 deletions.
2 changes: 1 addition & 1 deletion Mathlib/Data/Finset/NoncommProd.lean
Expand Up @@ -51,7 +51,7 @@ def noncommFoldr (s : Multiset α)
@[simp]
theorem noncommFoldr_coe (l : List α) (comm) (b : β) :
noncommFoldr f (l : Multiset α) comm b = l.foldr f b := by
simp only [noncommFoldr, coe_foldr, coe_attach, List.attach, Function.comp]
simp only [noncommFoldr, coe_foldr, coe_attach, List.attach, List.attachWith, Function.comp]
rw [← List.foldr_map]
simp [List.map_pmap, List.pmap_eq_map]
#align multiset.noncomm_foldr_coe Multiset.noncommFoldr_coe
Expand Down
4 changes: 2 additions & 2 deletions Mathlib/Data/List/Basic.lean
Expand Up @@ -2646,13 +2646,13 @@ theorem pmap_map {p : β → Prop} (g : ∀ b, p b → γ) (f : α → β) (l H)

theorem pmap_eq_map_attach {p : α → Prop} (f : ∀ a, p a → β) (l H) :
pmap f l H = l.attach.map fun x => f x.1 (H _ x.2) := by
rw [attach, map_pmap]; exact pmap_congr l fun _ _ _ _ => rfl
rw [attach, attachWith, map_pmap]; exact pmap_congr l fun _ _ _ _ => rfl
#align list.pmap_eq_map_attach List.pmap_eq_map_attach

-- @[simp] -- Porting note (#10959): lean 4 simp can't rewrite with this
theorem attach_map_coe' (l : List α) (f : α → β) :
(l.attach.map fun (i : {i // i ∈ l}) => f i) = l.map f := by
rw [attach, map_pmap]; exact pmap_eq_map _ _ _ _
rw [attach, attachWith, map_pmap]; exact pmap_eq_map _ _ _ _
#align list.attach_map_coe' List.attach_map_coe'

theorem attach_map_val' (l : List α) (f : α → β) : (l.attach.map fun i => f i.val) = l.map f :=
Expand Down
2 changes: 0 additions & 2 deletions Mathlib/Logic/Function/Basic.lean
Expand Up @@ -69,8 +69,6 @@ lemma hfunext {α α' : Sort u} {β : α → Sort v} {β' : α' → Sort v} {f :
exact eq_of_heq (this a)
#align function.hfunext Function.hfunext

theorem funext_iff {β : α → Sort*} {f₁ f₂ : ∀ x : α, β x} : f₁ = f₂ ↔ ∀ a, f₁ a = f₂ a :=
Iff.intro (fun h _ ↦ h ▸ rfl) funext
#align function.funext_iff Function.funext_iff

theorem ne_iff {β : α → Sort*} {f₁ f₂ : ∀ a, β a} : f₁ ≠ f₂ ↔ ∃ a, f₁ a ≠ f₂ a :=
Expand Down
2 changes: 1 addition & 1 deletion lake-manifest.json
Expand Up @@ -4,7 +4,7 @@
[{"url": "https://github.com/leanprover/std4",
"type": "git",
"subDir": null,
"rev": "32983874c1b897d78f20d620fe92fc8fd3f06c3a",
"rev": "cb172855f1712a9e906e91f3e14541960562fb78",
"name": "std",
"manifestFile": "lake-manifest.json",
"inputRev": "main",
Expand Down
1 change: 1 addition & 0 deletions scripts/noshake.json
Expand Up @@ -329,6 +329,7 @@
"Mathlib.Data.List.Lemmas": ["Mathlib.Data.List.InsertNth"],
"Mathlib.Data.List.EditDistance.Defs": ["Mathlib.Algebra.Ring.Nat"],
"Mathlib.Data.List.Basic": ["Mathlib.Data.Option.Basic", "Mathlib.Init.Core"],
"Mathlib.Data.FunLike.Basic": ["Mathlib.Logic.Function.Basic"],
"Mathlib.Data.Finset.Basic": ["Mathlib.Data.Finset.Attr"],
"Mathlib.Control.Traversable.Instances": ["Mathlib.Control.Applicative"],
"Mathlib.Control.Monad.Basic": ["Mathlib.Init.Control.Lawful"],
Expand Down

0 comments on commit dc34930

Please sign in to comment.