Skip to content

Commit

Permalink
Bump mathlib
Browse files Browse the repository at this point in the history
  • Loading branch information
YaelDillies committed Dec 29, 2024
1 parent 11de551 commit 30ad8bf
Show file tree
Hide file tree
Showing 4 changed files with 2 additions and 23 deletions.
1 change: 0 additions & 1 deletion LeanCamCombi.lean
Original file line number Diff line number Diff line change
Expand Up @@ -36,7 +36,6 @@ import LeanCamCombi.Mathlib.Algebra.MvPolynomial.Basic
import LeanCamCombi.Mathlib.Algebra.MvPolynomial.Degrees
import LeanCamCombi.Mathlib.Algebra.MvPolynomial.Equiv
import LeanCamCombi.Mathlib.Algebra.Order.Monoid.Unbundled.Pow
import LeanCamCombi.Mathlib.Algebra.Polynomial.CoeffMem
import LeanCamCombi.Mathlib.Algebra.Polynomial.Degree.Lemmas
import LeanCamCombi.Mathlib.Algebra.Ring.Hom.Defs
import LeanCamCombi.Mathlib.AlgebraicGeometry.PrimeSpectrum.Basic
Expand Down
3 changes: 1 addition & 2 deletions LeanCamCombi/GrowthInGroups/ChevalleyComplex.lean
Original file line number Diff line number Diff line change
Expand Up @@ -6,7 +6,6 @@ import LeanCamCombi.Mathlib.Algebra.MvPolynomial.Basic
import LeanCamCombi.Mathlib.Algebra.MvPolynomial.Degrees
import LeanCamCombi.Mathlib.Algebra.MvPolynomial.Equiv
import LeanCamCombi.Mathlib.Algebra.Order.Monoid.Unbundled.Pow
import LeanCamCombi.Mathlib.Algebra.Polynomial.CoeffMem
import LeanCamCombi.Mathlib.Algebra.Polynomial.Degree.Lemmas
import LeanCamCombi.Mathlib.AlgebraicGeometry.PrimeSpectrum.Basic
import LeanCamCombi.Mathlib.Data.Prod.Lex
Expand Down Expand Up @@ -375,7 +374,7 @@ lemma isConstructible_comap_C_zeroLocus_sdiff_zeroLocus :
obtain ⟨S, hS, hS'⟩ := H f
refine ⟨S, Eq.trans ?_ hS, ?_⟩
· rw [← zeroLocus_span (Set.range _), ← zeroLocus_span (Set.range _),
idealSpan_range_update_divByMonic hne hi]
idealSpan_range_update_divByMonic hne _ hi]
· intro C hC
let c' : InductionObj _ _ := ⟨Function.update c.val j (c.val j %ₘ c.val i)⟩
have deg_bound₁ : c'.degBound ≤ c.degBound := by
Expand Down
19 changes: 0 additions & 19 deletions LeanCamCombi/Mathlib/Algebra/Polynomial/CoeffMem.lean

This file was deleted.

2 changes: 1 addition & 1 deletion lake-manifest.json
Original file line number Diff line number Diff line change
Expand Up @@ -15,7 +15,7 @@
"type": "git",
"subDir": null,
"scope": "",
"rev": "68fbd252aa5d0168c5f582c0f66b3005dba683e1",
"rev": "3f703ecb9714a08b92a17f9c3c19ffc32343fede",
"name": "mathlib",
"manifestFile": "lake-manifest.json",
"inputRev": null,
Expand Down

0 comments on commit 30ad8bf

Please sign in to comment.