Skip to content

Commit

Permalink
chore: adaptations for nightly-2024-09-24 (#17094)
Browse files Browse the repository at this point in the history
Co-authored-by: leanprover-community-mathlib4-bot <[email protected]>
Co-authored-by: Kim Morrison <[email protected]>
  • Loading branch information
3 people committed Sep 24, 2024
1 parent c1c183a commit 84b2784
Show file tree
Hide file tree
Showing 5 changed files with 4 additions and 12 deletions.
1 change: 0 additions & 1 deletion Mathlib/Algebra/AddTorsor.lean
Original file line number Diff line number Diff line change
Expand Up @@ -248,7 +248,6 @@ instance instAddTorsor : AddTorsor (G × G') (P × P') where
zero_vadd _ := Prod.ext (zero_vadd _ _) (zero_vadd _ _)
add_vadd _ _ _ := Prod.ext (add_vadd _ _ _) (add_vadd _ _ _)
vsub p₁ p₂ := (p₁.1 -ᵥ p₂.1, p₁.2 -ᵥ p₂.2)
nonempty := Prod.instNonempty
vsub_vadd' _ _ := Prod.ext (vsub_vadd _ _) (vsub_vadd _ _)
vadd_vsub' _ _ := Prod.ext (vadd_vsub _ _) (vadd_vsub _ _)

Expand Down
7 changes: 0 additions & 7 deletions Mathlib/Logic/Nonempty.lean
Original file line number Diff line number Diff line change
Expand Up @@ -99,13 +99,6 @@ theorem Nonempty.elim_to_inhabited {α : Sort*} [h : Nonempty α] {p : Prop} (f
p :=
h.elim <| f ∘ Inhabited.mk

protected instance Prod.instNonempty {α β} [h : Nonempty α] [h2 : Nonempty β] : Nonempty (α × β) :=
h.elim fun g ↦ h2.elim fun g2 ↦ ⟨⟨g, g2⟩⟩

protected instance Pi.instNonempty {ι : Sort*} {α : ι → Sort*} [∀ i, Nonempty (α i)] :
Nonempty (∀ i, α i) :=
fun _ ↦ Classical.arbitrary _⟩

theorem Classical.nonempty_pi {ι} {α : ι → Sort*} : Nonempty (∀ i, α i) ↔ ∀ i, Nonempty (α i) :=
fun ⟨f⟩ a ↦ ⟨f a⟩, @Pi.instNonempty _ _⟩

Expand Down
4 changes: 2 additions & 2 deletions Mathlib/Topology/UniformSpace/UniformConvergenceTopology.lean
Original file line number Diff line number Diff line change
Expand Up @@ -157,9 +157,9 @@ open UniformConvergence

variable {α β : Type*} {𝔖 : Set (Set α)}

instance [Nonempty β] : Nonempty (α →ᵤ β) := Pi.instNonempty
instance [Nonempty β] : Nonempty (α →ᵤ β) := Pi.instNonempty _

instance [Nonempty β] : Nonempty (α →ᵤ[𝔖] β) := Pi.instNonempty
instance [Nonempty β] : Nonempty (α →ᵤ[𝔖] β) := Pi.instNonempty _

instance [Subsingleton β] : Subsingleton (α →ᵤ β) :=
inferInstanceAs <| Subsingleton <| α → β
Expand Down
2 changes: 1 addition & 1 deletion lake-manifest.json
Original file line number Diff line number Diff line change
Expand Up @@ -5,7 +5,7 @@
"type": "git",
"subDir": null,
"scope": "leanprover-community",
"rev": "6823ca35a23905867f0c6d9678932e6f261157e4",
"rev": "c37494a698d68c5e3711575fcb90ebf2974900ff",
"name": "batteries",
"manifestFile": "lake-manifest.json",
"inputRev": "nightly-testing",
Expand Down
2 changes: 1 addition & 1 deletion lean-toolchain
Original file line number Diff line number Diff line change
@@ -1 +1 @@
leanprover/lean4:nightly-2024-09-23
leanprover/lean4:nightly-2024-09-24

0 comments on commit 84b2784

Please sign in to comment.