Skip to content

Commit

Permalink
Merge branch 'master' into acmepjz_field_lin_disj
Browse files Browse the repository at this point in the history
  • Loading branch information
acmepjz committed Dec 2, 2024
2 parents 7c528b8 + 1e85f24 commit 6d4f500
Show file tree
Hide file tree
Showing 493 changed files with 10,295 additions and 4,743 deletions.
3 changes: 2 additions & 1 deletion .github/dependabot.yml
Original file line number Diff line number Diff line change
Expand Up @@ -3,7 +3,8 @@ version: 2 # Specifies the version of the Dependabot configuration file format
updates:
# Configuration for dependency updates
- package-ecosystem: "github-actions" # Specifies the ecosystem to check for updates
directory: "/" # Specifies the directory to check for dependencies; "/" means the root directory
directories:
- "/.github/*" # covers `build.in.yml` as well, which is not in `.github/workflows/` because it shouldn't be run in CI.
schedule:
# Check for updates to GitHub Actions every month
interval: "monthly"
34 changes: 34 additions & 0 deletions .github/workflows/zulip_emoji_awaiting_author.yaml
Original file line number Diff line number Diff line change
@@ -0,0 +1,34 @@
on:
pull_request:
types: [labeled, unlabeled]
jobs:
set_pr_emoji:
if: github.event.label.name == 'awaiting-author'
runs-on: ubuntu-latest
steps:
- name: Checkout mathlib repository
uses: actions/checkout@v4
with:
sparse-checkout: |
scripts/zulip_emoji_merge_delegate.py
- name: Set up Python
uses: actions/setup-python@v5
with:
python-version: '3.x'

- name: Install dependencies
run: |
python -m pip install --upgrade pip
pip install zulip
- name: Add or remove emoji
env:
ZULIP_API_KEY: ${{ secrets.ZULIP_API_KEY }}
ZULIP_EMAIL: [email protected]
ZULIP_SITE: https://leanprover.zulipchat.com
PR_NUMBER: ${{ github.event.number}}
LABEL_STATUS: ${{ github.event.action }}
run: |
printf $'Running the python script with pr "%s"\n' "$PR_NUMBER"
python scripts/zulip_emoji_merge_delegate.py "$ZULIP_API_KEY" "$ZULIP_EMAIL" "$ZULIP_SITE" "$LABEL_STATUS" "$PR_NUMBER"
14 changes: 7 additions & 7 deletions Archive/Imo/Imo2024Q5.lean
Original file line number Diff line number Diff line change
Expand Up @@ -229,7 +229,7 @@ lemma find?_eq_eq_find?_le {l : List (Cell N)} {r : Fin (N + 2)} (hne : l ≠ []
by_cases h : head.1 = r
· simp [h]
· have h' : ¬(r ≤ head.1) := fun hr' ↦ h (le_antisymm hf hr')
simp only [h, decide_False, Bool.false_eq_true, not_false_eq_true, List.find?_cons_of_neg, h']
simp only [h, decide_false, Bool.false_eq_true, not_false_eq_true, List.find?_cons_of_neg, h']
rcases tail with ⟨⟩ | ⟨htail, ttail⟩
· simp
· simp only [List.chain'_cons] at ha
Expand Down Expand Up @@ -315,7 +315,7 @@ lemma Path.tail_findFstEq (p : Path N) {r : Fin (N + 2)} (hr : r ≠ 0) :
rcases cells with ⟨⟩ | ⟨head, tail⟩
· simp at nonempty
· simp only [List.head_cons] at head_first_row
simp only [List.find?_cons, head_first_row, hr.symm, decide_False]
simp only [List.find?_cons, head_first_row, hr.symm, decide_false]
rfl
· simp_rw [Path.tail, if_neg h]

Expand All @@ -329,7 +329,7 @@ lemma Path.tail_firstMonster (p : Path N) (m : MonsterData N) :
· simp at nonempty
· simp only [List.head_cons] at head_first_row
simp only [List.find?_cons, head_first_row,
m.not_mem_monsterCells_of_fst_eq_zero head_first_row, decide_False]
m.not_mem_monsterCells_of_fst_eq_zero head_first_row, decide_false]
rfl
· simp_rw [Path.tail, if_neg h]

Expand All @@ -352,17 +352,17 @@ lemma Path.firstMonster_eq_of_findFstEq_mem {p : Path N} {m : MonsterData N}
· simp only [List.head_cons] at head_first_row
simp only [List.getElem_cons_succ] at h1
simp only [List.length_cons, lt_add_iff_pos_left, List.length_pos_iff_ne_nil] at hl
simp only [m.not_mem_monsterCells_of_fst_eq_zero head_first_row, decide_False,
simp only [m.not_mem_monsterCells_of_fst_eq_zero head_first_row, decide_false,
Bool.false_eq_true, not_false_eq_true, List.find?_cons_of_neg, head_first_row,
Fin.zero_eq_one_iff, Nat.reduceEqDiff, Option.some_get]
simp only [findFstEq, head_first_row, Fin.zero_eq_one_iff, Nat.reduceEqDiff, decide_False,
simp only [findFstEq, head_first_row, Fin.zero_eq_one_iff, Nat.reduceEqDiff, decide_false,
Bool.false_eq_true, not_false_eq_true, List.find?_cons_of_neg] at h
rcases tail with ⟨⟩ | ⟨htail, ttail⟩
· simp at hl
· simp only [List.getElem_cons_zero] at h1
have h1' : htail.1 = 1 := by simp [Fin.ext_iff, h1]
simp only [h1', decide_True, List.find?_cons_of_pos, Option.get_some] at h
simp only [h1', h, decide_True, List.find?_cons_of_pos]
simp only [h1', decide_true, List.find?_cons_of_pos, Option.get_some] at h
simp only [h1', h, decide_true, List.find?_cons_of_pos]
case ind p ht =>
have h1 : (1 : Fin (N + 2)) ≠ 0 := by simp
rw [p.tail_findFstEq h1, p.tail_firstMonster m] at ht
Expand Down
4 changes: 1 addition & 3 deletions Archive/MiuLanguage/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -106,9 +106,7 @@ instance : Repr MiuAtom :=

/-- For simplicity, an `Miustr` is just a list of elements of type `MiuAtom`.
-/
def Miustr :=
List MiuAtom
deriving Append
abbrev Miustr := List MiuAtom

instance : Membership MiuAtom Miustr := by unfold Miustr; infer_instance

Expand Down
9 changes: 2 additions & 7 deletions Counterexamples/HomogeneousPrimeNotPrime.lean
Original file line number Diff line number Diff line change
Expand Up @@ -110,13 +110,8 @@ theorem grading.right_inv : Function.RightInverse (coeLinearMap (grading R)) gra
induction' zz using DirectSum.induction_on with i zz d1 d2 ih1 ih2
· simp only [map_zero]
· rcases i with (_ | ⟨⟨⟩⟩) <;> rcases zz with ⟨⟨a, b⟩, hab : _ = _⟩ <;> dsimp at hab <;>
cases hab <;>
-- Porting note: proof was `decide`
-- now we need a `simp` and two `erw` subproofs...
simp only [coeLinearMap_of, decompose, AddMonoidHom.coe_mk,
ZeroHom.coe_mk, sub_self, sub_zero]
· erw [map_zero (of (grading R ·) 1), add_zero]; rfl
· erw [map_zero (of (grading R ·) 0), zero_add]; rfl
-- Porting note: proof was `decide` (without reverting any free variables).
cases hab <;> decide +revert
· simp only [map_add, ih1, ih2]

theorem grading.left_inv : Function.LeftInverse (coeLinearMap (grading R)) grading.decompose :=
Expand Down
42 changes: 37 additions & 5 deletions Mathlib.lean
Original file line number Diff line number Diff line change
Expand Up @@ -153,6 +153,7 @@ import Mathlib.Algebra.Category.Ring.Instances
import Mathlib.Algebra.Category.Ring.Limits
import Mathlib.Algebra.Category.Ring.LinearAlgebra
import Mathlib.Algebra.Category.Ring.Under.Basic
import Mathlib.Algebra.Category.Ring.Under.Limits
import Mathlib.Algebra.Category.Semigrp.Basic
import Mathlib.Algebra.Central.Basic
import Mathlib.Algebra.Central.Defs
Expand Down Expand Up @@ -201,6 +202,7 @@ import Mathlib.Algebra.DirectSum.LinearMap
import Mathlib.Algebra.DirectSum.Module
import Mathlib.Algebra.DirectSum.Ring
import Mathlib.Algebra.Divisibility.Basic
import Mathlib.Algebra.Divisibility.Hom
import Mathlib.Algebra.Divisibility.Prod
import Mathlib.Algebra.Divisibility.Units
import Mathlib.Algebra.DualNumber
Expand Down Expand Up @@ -319,6 +321,7 @@ import Mathlib.Algebra.Group.Subgroup.Pointwise
import Mathlib.Algebra.Group.Subgroup.ZPowers.Basic
import Mathlib.Algebra.Group.Subgroup.ZPowers.Lemmas
import Mathlib.Algebra.Group.Submonoid.Basic
import Mathlib.Algebra.Group.Submonoid.BigOperators
import Mathlib.Algebra.Group.Submonoid.Defs
import Mathlib.Algebra.Group.Submonoid.DistribMulAction
import Mathlib.Algebra.Group.Submonoid.Membership
Expand Down Expand Up @@ -404,6 +407,7 @@ import Mathlib.Algebra.Homology.DifferentialObject
import Mathlib.Algebra.Homology.Embedding.Basic
import Mathlib.Algebra.Homology.Embedding.Boundary
import Mathlib.Algebra.Homology.Embedding.Extend
import Mathlib.Algebra.Homology.Embedding.ExtendHomology
import Mathlib.Algebra.Homology.Embedding.HomEquiv
import Mathlib.Algebra.Homology.Embedding.IsSupported
import Mathlib.Algebra.Homology.Embedding.Restriction
Expand Down Expand Up @@ -615,6 +619,7 @@ import Mathlib.Algebra.Order.AddGroupWithTop
import Mathlib.Algebra.Order.AddTorsor
import Mathlib.Algebra.Order.Algebra
import Mathlib.Algebra.Order.Antidiag.Finsupp
import Mathlib.Algebra.Order.Antidiag.Nat
import Mathlib.Algebra.Order.Antidiag.Pi
import Mathlib.Algebra.Order.Antidiag.Prod
import Mathlib.Algebra.Order.Archimedean.Basic
Expand Down Expand Up @@ -941,8 +946,9 @@ import Mathlib.AlgebraicGeometry.EllipticCurve.Affine
import Mathlib.AlgebraicGeometry.EllipticCurve.DivisionPolynomial.Basic
import Mathlib.AlgebraicGeometry.EllipticCurve.DivisionPolynomial.Degree
import Mathlib.AlgebraicGeometry.EllipticCurve.Group
import Mathlib.AlgebraicGeometry.EllipticCurve.J
import Mathlib.AlgebraicGeometry.EllipticCurve.IsomOfJ
import Mathlib.AlgebraicGeometry.EllipticCurve.Jacobian
import Mathlib.AlgebraicGeometry.EllipticCurve.ModelsWithJ
import Mathlib.AlgebraicGeometry.EllipticCurve.NormalForms
import Mathlib.AlgebraicGeometry.EllipticCurve.Projective
import Mathlib.AlgebraicGeometry.EllipticCurve.VariableChange
Expand Down Expand Up @@ -1004,6 +1010,7 @@ import Mathlib.AlgebraicGeometry.Scheme
import Mathlib.AlgebraicGeometry.Sites.BigZariski
import Mathlib.AlgebraicGeometry.Sites.Etale
import Mathlib.AlgebraicGeometry.Sites.MorphismProperty
import Mathlib.AlgebraicGeometry.Sites.Small
import Mathlib.AlgebraicGeometry.Spec
import Mathlib.AlgebraicGeometry.SpreadingOut
import Mathlib.AlgebraicGeometry.Stalk
Expand Down Expand Up @@ -1125,7 +1132,6 @@ import Mathlib.Analysis.Calculus.BumpFunction.InnerProduct
import Mathlib.Analysis.Calculus.BumpFunction.Normed
import Mathlib.Analysis.Calculus.Conformal.InnerProduct
import Mathlib.Analysis.Calculus.Conformal.NormedSpace
import Mathlib.Analysis.Calculus.ContDiff.Analytic
import Mathlib.Analysis.Calculus.ContDiff.Basic
import Mathlib.Analysis.Calculus.ContDiff.Bounds
import Mathlib.Analysis.Calculus.ContDiff.CPolynomial
Expand Down Expand Up @@ -1619,6 +1625,7 @@ import Mathlib.CategoryTheory.Category.Basic
import Mathlib.CategoryTheory.Category.Bipointed
import Mathlib.CategoryTheory.Category.Cat
import Mathlib.CategoryTheory.Category.Cat.Adjunction
import Mathlib.CategoryTheory.Category.Cat.AsSmall
import Mathlib.CategoryTheory.Category.Cat.Limit
import Mathlib.CategoryTheory.Category.Factorisation
import Mathlib.CategoryTheory.Category.GaloisConnection
Expand Down Expand Up @@ -2123,6 +2130,8 @@ import Mathlib.CategoryTheory.Sites.Whiskering
import Mathlib.CategoryTheory.Skeletal
import Mathlib.CategoryTheory.SmallObject.Construction
import Mathlib.CategoryTheory.SmallObject.Iteration.Basic
import Mathlib.CategoryTheory.SmallObject.Iteration.ExtendToSucc
import Mathlib.CategoryTheory.SmallObject.Iteration.Nonempty
import Mathlib.CategoryTheory.SmallObject.Iteration.UniqueHom
import Mathlib.CategoryTheory.Square
import Mathlib.CategoryTheory.Subobject.Basic
Expand Down Expand Up @@ -2196,6 +2205,7 @@ import Mathlib.Combinatorics.Quiver.Cast
import Mathlib.Combinatorics.Quiver.ConnectedComponent
import Mathlib.Combinatorics.Quiver.Covering
import Mathlib.Combinatorics.Quiver.Path
import Mathlib.Combinatorics.Quiver.Prefunctor
import Mathlib.Combinatorics.Quiver.Push
import Mathlib.Combinatorics.Quiver.ReflQuiver
import Mathlib.Combinatorics.Quiver.SingleObj
Expand Down Expand Up @@ -2381,6 +2391,7 @@ import Mathlib.Data.ENNReal.Operations
import Mathlib.Data.ENNReal.Real
import Mathlib.Data.ENat.Basic
import Mathlib.Data.ENat.BigOperators
import Mathlib.Data.ENat.Defs
import Mathlib.Data.ENat.Lattice
import Mathlib.Data.Erased
import Mathlib.Data.FP.Basic
Expand Down Expand Up @@ -2759,6 +2770,7 @@ import Mathlib.Data.PNat.Equiv
import Mathlib.Data.PNat.Factors
import Mathlib.Data.PNat.Find
import Mathlib.Data.PNat.Interval
import Mathlib.Data.PNat.Notation
import Mathlib.Data.PNat.Prime
import Mathlib.Data.PNat.Xgcd
import Mathlib.Data.PSigma.Order
Expand Down Expand Up @@ -3062,6 +3074,7 @@ import Mathlib.Geometry.Manifold.MFDeriv.Atlas
import Mathlib.Geometry.Manifold.MFDeriv.Basic
import Mathlib.Geometry.Manifold.MFDeriv.Defs
import Mathlib.Geometry.Manifold.MFDeriv.FDeriv
import Mathlib.Geometry.Manifold.MFDeriv.NormedSpace
import Mathlib.Geometry.Manifold.MFDeriv.SpecificFunctions
import Mathlib.Geometry.Manifold.MFDeriv.Tangent
import Mathlib.Geometry.Manifold.MFDeriv.UniqueDifferential
Expand Down Expand Up @@ -3128,6 +3141,7 @@ import Mathlib.GroupTheory.FreeGroup.Basic
import Mathlib.GroupTheory.FreeGroup.IsFreeGroup
import Mathlib.GroupTheory.FreeGroup.NielsenSchreier
import Mathlib.GroupTheory.FreeGroup.Reduce
import Mathlib.GroupTheory.Goursat
import Mathlib.GroupTheory.GroupAction.Basic
import Mathlib.GroupTheory.GroupAction.Blocks
import Mathlib.GroupTheory.GroupAction.CardCommute
Expand Down Expand Up @@ -3346,6 +3360,7 @@ import Mathlib.LinearAlgebra.LinearIndependent
import Mathlib.LinearAlgebra.LinearPMap
import Mathlib.LinearAlgebra.Matrix.AbsoluteValue
import Mathlib.LinearAlgebra.Matrix.Adjugate
import Mathlib.LinearAlgebra.Matrix.BaseChange
import Mathlib.LinearAlgebra.Matrix.Basis
import Mathlib.LinearAlgebra.Matrix.BilinearForm
import Mathlib.LinearAlgebra.Matrix.Block
Expand Down Expand Up @@ -3747,6 +3762,7 @@ import Mathlib.ModelTheory.Syntax
import Mathlib.ModelTheory.Types
import Mathlib.ModelTheory.Ultraproducts
import Mathlib.NumberTheory.ADEInequality
import Mathlib.NumberTheory.AbelSummation
import Mathlib.NumberTheory.ArithmeticFunction
import Mathlib.NumberTheory.Basic
import Mathlib.NumberTheory.Bernoulli
Expand Down Expand Up @@ -4094,6 +4110,7 @@ import Mathlib.Order.Sublattice
import Mathlib.Order.SuccPred.Archimedean
import Mathlib.Order.SuccPred.Basic
import Mathlib.Order.SuccPred.CompleteLinearOrder
import Mathlib.Order.SuccPred.InitialSeg
import Mathlib.Order.SuccPred.IntervalSucc
import Mathlib.Order.SuccPred.Limit
import Mathlib.Order.SuccPred.LinearLocallyFinite
Expand Down Expand Up @@ -4198,13 +4215,24 @@ import Mathlib.RingTheory.Adjoin.Basic
import Mathlib.RingTheory.Adjoin.Dimension
import Mathlib.RingTheory.Adjoin.FG
import Mathlib.RingTheory.Adjoin.Field
import Mathlib.RingTheory.Adjoin.Polynomial
import Mathlib.RingTheory.Adjoin.PowerBasis
import Mathlib.RingTheory.Adjoin.Tower
import Mathlib.RingTheory.AdjoinRoot
import Mathlib.RingTheory.AlgebraTower
import Mathlib.RingTheory.Algebraic
import Mathlib.RingTheory.Algebraic.Basic
import Mathlib.RingTheory.Algebraic.Cardinality
import Mathlib.RingTheory.AlgebraicIndependent
import Mathlib.RingTheory.Algebraic.Defs
import Mathlib.RingTheory.Algebraic.Integral
import Mathlib.RingTheory.Algebraic.LinearIndependent
import Mathlib.RingTheory.Algebraic.MvPolynomial
import Mathlib.RingTheory.Algebraic.Pi
import Mathlib.RingTheory.AlgebraicIndependent.Adjoin
import Mathlib.RingTheory.AlgebraicIndependent.Basic
import Mathlib.RingTheory.AlgebraicIndependent.Defs
import Mathlib.RingTheory.AlgebraicIndependent.RankAndCardinality
import Mathlib.RingTheory.AlgebraicIndependent.TranscendenceBasis
import Mathlib.RingTheory.AlgebraicIndependent.Transcendental
import Mathlib.RingTheory.Artinian
import Mathlib.RingTheory.Bezout
import Mathlib.RingTheory.Bialgebra.Basic
Expand Down Expand Up @@ -4412,6 +4440,7 @@ import Mathlib.RingTheory.MvPowerSeries.Inverse
import Mathlib.RingTheory.MvPowerSeries.LexOrder
import Mathlib.RingTheory.MvPowerSeries.NoZeroDivisors
import Mathlib.RingTheory.MvPowerSeries.Order
import Mathlib.RingTheory.MvPowerSeries.PiTopology
import Mathlib.RingTheory.MvPowerSeries.Trunc
import Mathlib.RingTheory.Nakayama
import Mathlib.RingTheory.Nilpotent.Basic
Expand Down Expand Up @@ -4452,6 +4481,7 @@ import Mathlib.RingTheory.Polynomial.Eisenstein.IsIntegral
import Mathlib.RingTheory.Polynomial.GaussLemma
import Mathlib.RingTheory.Polynomial.Hermite.Basic
import Mathlib.RingTheory.Polynomial.Hermite.Gaussian
import Mathlib.RingTheory.Polynomial.Ideal
import Mathlib.RingTheory.Polynomial.IntegralNormalization
import Mathlib.RingTheory.Polynomial.IrreducibleRing
import Mathlib.RingTheory.Polynomial.Nilpotent
Expand All @@ -4473,6 +4503,7 @@ import Mathlib.RingTheory.PowerSeries.Basic
import Mathlib.RingTheory.PowerSeries.Derivative
import Mathlib.RingTheory.PowerSeries.Inverse
import Mathlib.RingTheory.PowerSeries.Order
import Mathlib.RingTheory.PowerSeries.PiTopology
import Mathlib.RingTheory.PowerSeries.Trunc
import Mathlib.RingTheory.PowerSeries.WellKnown
import Mathlib.RingTheory.Presentation
Expand Down Expand Up @@ -4517,6 +4548,7 @@ import Mathlib.RingTheory.TensorProduct.Basic
import Mathlib.RingTheory.TensorProduct.Finite
import Mathlib.RingTheory.TensorProduct.Free
import Mathlib.RingTheory.TensorProduct.MvPolynomial
import Mathlib.RingTheory.TensorProduct.Pi
import Mathlib.RingTheory.Trace.Basic
import Mathlib.RingTheory.Trace.Defs
import Mathlib.RingTheory.Trace.Quotient
Expand Down Expand Up @@ -4972,6 +5004,7 @@ import Mathlib.Topology.Algebra.SeparationQuotient.Basic
import Mathlib.Topology.Algebra.SeparationQuotient.Section
import Mathlib.Topology.Algebra.Star
import Mathlib.Topology.Algebra.StarSubalgebra
import Mathlib.Topology.Algebra.Support
import Mathlib.Topology.Algebra.UniformConvergence
import Mathlib.Topology.Algebra.UniformField
import Mathlib.Topology.Algebra.UniformFilterBasis
Expand Down Expand Up @@ -5304,7 +5337,6 @@ import Mathlib.Topology.Sober
import Mathlib.Topology.Specialization
import Mathlib.Topology.Spectral.Hom
import Mathlib.Topology.StoneCech
import Mathlib.Topology.Support
import Mathlib.Topology.TietzeExtension
import Mathlib.Topology.Ultrafilter
import Mathlib.Topology.UniformSpace.AbsoluteValue
Expand Down
Loading

0 comments on commit 6d4f500

Please sign in to comment.