Skip to content

Commit 0bf03c5

Browse files
committed
chore: more cancelling pairs (#34051)
Found by the linter at #34024.
1 parent 80046e6 commit 0bf03c5

File tree

4 files changed

+0
-17
lines changed

4 files changed

+0
-17
lines changed

Mathlib/Algebra/Ring/Units.lean

Lines changed: 0 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -138,5 +138,3 @@ theorem isUnit_map (f : α →+* β) {a : α} : IsUnit a → IsUnit (f a) :=
138138
end Semiring
139139

140140
end RingHom
141-
142-
variable [Semiring α] [Semiring β]

Mathlib/Analysis/Normed/Order/Basic.lean

Lines changed: 0 additions & 9 deletions
Original file line numberDiff line numberDiff line change
@@ -13,12 +13,3 @@ public import Mathlib.Analysis.Normed.Group.Basic
1313
In this file, we define classes for fields and groups that are both normed and ordered.
1414
These are mostly useful to avoid diamonds during type class inference.
1515
-/
16-
17-
public section
18-
19-
20-
open Filter Set
21-
22-
open Topology
23-
24-
variable {α : Type*}

Mathlib/Data/Matrix/Basic.lean

Lines changed: 0 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -928,8 +928,6 @@ def transposeAlgEquiv [CommSemiring R] [CommSemiring α] [Fintype m] [DecidableE
928928
commutes' := fun r => by
929929
simp only [algebraMap_eq_diagonal, diagonal_transpose, MulOpposite.algebraMap_apply] }
930930

931-
variable {R m α}
932-
933931
end Transpose
934932

935933
section NonUnitalNonAssocSemiring

Mathlib/Topology/Algebra/IsUniformGroup/Defs.lean

Lines changed: 0 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -150,8 +150,6 @@ theorem uniformity_eq_comap_nhds_one_swapped :
150150
rw [← comap_swap_uniformity, uniformity_eq_comap_nhds_one, comap_comap, Function.comp_def]
151151
simp
152152

153-
variable {Gₗ Gᵣ}
154-
155153
end LeftRight
156154

157155
section IsUniformGroup
@@ -412,8 +410,6 @@ theorem IsUniformGroup.uniformity_countably_generated [(𝓝 (1 : α)).IsCountab
412410
rw [uniformity_eq_comap_nhds_one]
413411
exact Filter.comap.isCountablyGenerated _ _
414412

415-
open MulOpposite
416-
417413
end
418414

419415
section OfLeftAndRight

0 commit comments

Comments
 (0)