Skip to content

Commit

Permalink
Browse files Browse the repository at this point in the history
  • Loading branch information
leanprover-community-mathlib4-bot committed Oct 25, 2024
2 parents 45e73ef + 1a5abab commit 5720c0f
Show file tree
Hide file tree
Showing 245 changed files with 2,991 additions and 2,175 deletions.
2 changes: 1 addition & 1 deletion Archive/Imo/Imo2019Q4.lean
Original file line number Diff line number Diff line change
Expand Up @@ -5,7 +5,7 @@ Authors: Floris van Doorn
-/
import Mathlib.Data.Nat.Factorial.BigOperators
import Mathlib.Data.Nat.Multiplicity
import Mathlib.Data.Nat.Prime.Basic
import Mathlib.Data.Nat.Prime.Int
import Mathlib.Tactic.IntervalCases
import Mathlib.Tactic.GCongr

Expand Down
24 changes: 19 additions & 5 deletions Mathlib.lean
Original file line number Diff line number Diff line change
Expand Up @@ -319,6 +319,8 @@ import Mathlib.Algebra.Group.ZeroOne
import Mathlib.Algebra.GroupPower.IterateHom
import Mathlib.Algebra.GroupWithZero.Action.Basic
import Mathlib.Algebra.GroupWithZero.Action.Defs
import Mathlib.Algebra.GroupWithZero.Action.End
import Mathlib.Algebra.GroupWithZero.Action.Faithful
import Mathlib.Algebra.GroupWithZero.Action.Opposite
import Mathlib.Algebra.GroupWithZero.Action.Pi
import Mathlib.Algebra.GroupWithZero.Action.Prod
Expand Down Expand Up @@ -769,6 +771,8 @@ import Mathlib.Algebra.Polynomial.Splits
import Mathlib.Algebra.Polynomial.SumIteratedDerivative
import Mathlib.Algebra.Polynomial.Taylor
import Mathlib.Algebra.Polynomial.UnitTrinomial
import Mathlib.Algebra.Prime.Defs
import Mathlib.Algebra.Prime.Lemmas
import Mathlib.Algebra.QuadraticDiscriminant
import Mathlib.Algebra.Quandle
import Mathlib.Algebra.Quaternion
Expand Down Expand Up @@ -1486,6 +1490,7 @@ import Mathlib.CategoryTheory.Bicategory.End
import Mathlib.CategoryTheory.Bicategory.Extension
import Mathlib.CategoryTheory.Bicategory.Free
import Mathlib.CategoryTheory.Bicategory.Functor.Lax
import Mathlib.CategoryTheory.Bicategory.Functor.LocallyDiscrete
import Mathlib.CategoryTheory.Bicategory.Functor.Oplax
import Mathlib.CategoryTheory.Bicategory.Functor.Prelax
import Mathlib.CategoryTheory.Bicategory.Functor.Pseudofunctor
Expand Down Expand Up @@ -1539,7 +1544,8 @@ import Mathlib.CategoryTheory.Comma.Basic
import Mathlib.CategoryTheory.Comma.Over
import Mathlib.CategoryTheory.Comma.Presheaf.Basic
import Mathlib.CategoryTheory.Comma.Presheaf.Colimit
import Mathlib.CategoryTheory.Comma.StructuredArrow
import Mathlib.CategoryTheory.Comma.StructuredArrow.Basic
import Mathlib.CategoryTheory.Comma.StructuredArrow.Small
import Mathlib.CategoryTheory.ComposableArrows
import Mathlib.CategoryTheory.ConcreteCategory.Basic
import Mathlib.CategoryTheory.ConcreteCategory.Bundled
Expand Down Expand Up @@ -1728,6 +1734,7 @@ import Mathlib.CategoryTheory.Limits.Shapes.FiniteProducts
import Mathlib.CategoryTheory.Limits.Shapes.FunctorCategory
import Mathlib.CategoryTheory.Limits.Shapes.FunctorToTypes
import Mathlib.CategoryTheory.Limits.Shapes.Images
import Mathlib.CategoryTheory.Limits.Shapes.IsTerminal
import Mathlib.CategoryTheory.Limits.Shapes.KernelPair
import Mathlib.CategoryTheory.Limits.Shapes.Kernels
import Mathlib.CategoryTheory.Limits.Shapes.Multiequalizer
Expand Down Expand Up @@ -2396,7 +2403,9 @@ import Mathlib.Data.List.NodupEquivFin
import Mathlib.Data.List.OfFn
import Mathlib.Data.List.Pairwise
import Mathlib.Data.List.Palindrome
import Mathlib.Data.List.Perm
import Mathlib.Data.List.Perm.Basic
import Mathlib.Data.List.Perm.Lattice
import Mathlib.Data.List.Perm.Subperm
import Mathlib.Data.List.Permutation
import Mathlib.Data.List.Pi
import Mathlib.Data.List.Prime
Expand Down Expand Up @@ -2535,6 +2544,10 @@ import Mathlib.Data.Nat.PartENat
import Mathlib.Data.Nat.Periodic
import Mathlib.Data.Nat.Prime.Basic
import Mathlib.Data.Nat.Prime.Defs
import Mathlib.Data.Nat.Prime.Factorial
import Mathlib.Data.Nat.Prime.Infinite
import Mathlib.Data.Nat.Prime.Int
import Mathlib.Data.Nat.Prime.Pow
import Mathlib.Data.Nat.PrimeFin
import Mathlib.Data.Nat.Set
import Mathlib.Data.Nat.Size
Expand Down Expand Up @@ -3792,7 +3805,6 @@ import Mathlib.Order.Interval.Set.SurjOn
import Mathlib.Order.Interval.Set.UnorderedInterval
import Mathlib.Order.Interval.Set.WithBotTop
import Mathlib.Order.Irreducible
import Mathlib.Order.IsWellOrderLimitElement
import Mathlib.Order.Iterate
import Mathlib.Order.JordanHolder
import Mathlib.Order.KonigLemma
Expand Down Expand Up @@ -4775,7 +4787,8 @@ import Mathlib.Topology.FiberBundle.IsHomeomorphicTrivialBundle
import Mathlib.Topology.FiberBundle.Trivialization
import Mathlib.Topology.FiberPartition
import Mathlib.Topology.Filter
import Mathlib.Topology.GDelta
import Mathlib.Topology.GDelta.Basic
import Mathlib.Topology.GDelta.UniformSpace
import Mathlib.Topology.Germ
import Mathlib.Topology.Gluing
import Mathlib.Topology.Hom.ContinuousEval
Expand Down Expand Up @@ -4923,7 +4936,8 @@ import Mathlib.Topology.QuasiSeparated
import Mathlib.Topology.RestrictGen
import Mathlib.Topology.Semicontinuous
import Mathlib.Topology.SeparatedMap
import Mathlib.Topology.Separation
import Mathlib.Topology.Separation.Basic
import Mathlib.Topology.Separation.GDelta
import Mathlib.Topology.Separation.NotNormal
import Mathlib.Topology.Sequences
import Mathlib.Topology.Sets.Closeds
Expand Down
1 change: 0 additions & 1 deletion Mathlib/Algebra/Algebra/Equiv.lean
Original file line number Diff line number Diff line change
Expand Up @@ -216,7 +216,6 @@ protected theorem map_mul : ∀ x y, e (x * y) = e x * e y :=
protected theorem map_one : e 1 = 1 :=
map_one e

-- @[simp] -- Porting note (#10618): simp can prove this
@[deprecated map_smul (since := "2024-06-20")]
protected theorem map_smul (r : R) (x : A₁) : e (r • x) = r • e x :=
map_smul _ _ _
Expand Down
1 change: 0 additions & 1 deletion Mathlib/Algebra/Algebra/Hom.lean
Original file line number Diff line number Diff line change
Expand Up @@ -218,7 +218,6 @@ protected theorem map_one : φ 1 = 1 :=
protected theorem map_pow (x : A) (n : ℕ) : φ (x ^ n) = φ x ^ n :=
map_pow _ _ _

-- @[simp] -- Porting note (#10618): simp can prove this
@[deprecated map_smul (since := "2024-06-26")]
protected theorem map_smul (r : R) (x : A) : φ (r • x) = r • φ x :=
map_smul _ _ _
Expand Down
3 changes: 0 additions & 3 deletions Mathlib/Algebra/Algebra/NonUnitalHom.lean
Original file line number Diff line number Diff line change
Expand Up @@ -245,15 +245,12 @@ theorem coe_mulHom_mk (f : A →ₛₙₐ[φ] B) (h₁ h₂ h₃ h₄) :
protected theorem map_smul (f : A →ₛₙₐ[φ] B) (c : R) (x : A) : f (c • x) = (φ c) • f x :=
map_smulₛₗ _ _ _

-- @[simp] -- Porting note (#10618) : simp can prove this
protected theorem map_add (f : A →ₛₙₐ[φ] B) (x y : A) : f (x + y) = f x + f y :=
map_add _ _ _

-- @[simp] -- Porting note (#10618) : simp can prove this
protected theorem map_mul (f : A →ₛₙₐ[φ] B) (x y : A) : f (x * y) = f x * f y :=
map_mul _ _ _

-- @[simp] -- Porting note (#10618) : simp can prove this
protected theorem map_zero (f : A →ₛₙₐ[φ] B) : f 0 = 0 :=
map_zero _

Expand Down
2 changes: 0 additions & 2 deletions Mathlib/Algebra/Algebra/Operations.lean
Original file line number Diff line number Diff line change
Expand Up @@ -184,12 +184,10 @@ theorem mul_bot : M * ⊥ = ⊥ :=
theorem bot_mul : ⊥ * M = ⊥ :=
map₂_bot_left _ _

-- @[simp] -- Porting note (#10618): simp can prove this once we have a monoid structure
protected theorem one_mul : (1 : Submodule R A) * M = M := by
conv_lhs => rw [one_eq_span, ← span_eq M]
erw [span_mul_span, one_mul, span_eq]

-- @[simp] -- Porting note (#10618): simp can prove this once we have a monoid structure
protected theorem mul_one : M * 1 = M := by
conv_lhs => rw [one_eq_span, ← span_eq M]
erw [span_mul_span, mul_one, span_eq]
Expand Down
1 change: 0 additions & 1 deletion Mathlib/Algebra/Algebra/Subalgebra/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -46,7 +46,6 @@ instance SubsemiringClass : SubsemiringClass (Subalgebra R A) A where
theorem mem_toSubsemiring {S : Subalgebra R A} {x} : x ∈ S.toSubsemiring ↔ x ∈ S :=
Iff.rfl

-- @[simp] -- Porting note (#10618): simp can prove this
theorem mem_carrier {s : Subalgebra R A} {x : A} : x ∈ s.carrier ↔ x ∈ s :=
Iff.rfl

Expand Down
Loading

0 comments on commit 5720c0f

Please sign in to comment.