Skip to content

Commit

Permalink
another batch
Browse files Browse the repository at this point in the history
  • Loading branch information
adomani committed Sep 29, 2024
1 parent a053d06 commit f70dfcd
Show file tree
Hide file tree
Showing 4 changed files with 8 additions and 9 deletions.
2 changes: 1 addition & 1 deletion Mathlib/Algebra/Module/BigOperators.lean
Original file line number Diff line number Diff line change
Expand Up @@ -15,7 +15,7 @@ variable {ι κ α β R M : Type*}

section AddCommMonoid

variable [Semiring R] [AddCommMonoid M] [Module R M] (r s : R) (x y : M)
variable [Semiring R] [AddCommMonoid M] [Module R M]

theorem List.sum_smul {l : List R} {x : M} : l.sum • x = (l.map fun r ↦ r • x).sum :=
map_list_sum ((smulAddHom R M).flip x) l
Expand Down
5 changes: 2 additions & 3 deletions Mathlib/Algebra/Polynomial/Induction.lean
Original file line number Diff line number Diff line change
Expand Up @@ -26,12 +26,11 @@ open Polynomial

universe u v w x y z

variable {R : Type u} {S : Type v} {T : Type w} {ι : Type x} {k : Type y} {A : Type z} {a b : R}
{m n : ℕ}
variable {R : Type u}

section Semiring

variable [Semiring R] {p q r : R[X]}
variable [Semiring R]

@[elab_as_elim]
protected theorem induction_on {M : R[X] → Prop} (p : R[X]) (h_C : ∀ a, M (C a))
Expand Down
8 changes: 4 additions & 4 deletions Mathlib/Order/Interval/Finset/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -683,7 +683,7 @@ variable [LinearOrder α]

section LocallyFiniteOrder

variable [LocallyFiniteOrder α] {a b : α}
variable [LocallyFiniteOrder α]

theorem Ico_subset_Ico_iff {a₁ b₁ a₂ b₂ : α} (h : a₁ < b₁) :
Ico a₁ b₁ ⊆ Ico a₂ b₂ ↔ a₂ ≤ a₁ ∧ b₁ ≤ b₂ := by
Expand Down Expand Up @@ -790,7 +790,7 @@ end LinearOrder

section Lattice

variable [Lattice α] [LocallyFiniteOrder α] {a a₁ a₂ b b₁ b₂ c x : α}
variable [Lattice α] [LocallyFiniteOrder α] {a a₁ a₂ b b₁ b₂ x : α}

theorem uIcc_toDual (a b : α) : [[toDual a, toDual b]] = [[a, b]].map toDual.toEmbedding :=
Icc_toDual _ _
Expand Down Expand Up @@ -862,7 +862,7 @@ end Lattice

section DistribLattice

variable [DistribLattice α] [LocallyFiniteOrder α] {a a₁ a₂ b b₁ b₂ c x : α}
variable [DistribLattice α] [LocallyFiniteOrder α] {a b c : α}

theorem eq_of_mem_uIcc_of_mem_uIcc : a ∈ [[b, c]] → b ∈ [[a, c]] → a = b := by
simp_rw [mem_uIcc]
Expand All @@ -883,7 +883,7 @@ end DistribLattice

section LinearOrder

variable [LinearOrder α] [LocallyFiniteOrder α] {a a₁ a₂ b b₁ b₂ c x : α}
variable [LinearOrder α] [LocallyFiniteOrder α] {a a₁ a₂ b b₁ b₂ c : α}

theorem Icc_min_max : Icc (min a b) (max a b) = [[a, b]] :=
rfl
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Order/SuccPred/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -927,7 +927,7 @@ lemma gc_pred_succ : GaloisConnection (pred : α → α) succ := fun _ _ ↦ pre

end Preorder

variable [PartialOrder α] [SuccOrder α] [PredOrder α] {a b : α}
variable [PartialOrder α] [SuccOrder α] [PredOrder α] {a : α}

@[simp]
theorem succ_pred_of_not_isMin (h : ¬IsMin a) : succ (pred a) = a :=
Expand Down

0 comments on commit f70dfcd

Please sign in to comment.