Skip to content

Commit f9bca0d

Browse files
chore: bump mathlib (#354)
* bump mathlib * Update FLT/AutomorphicRepresentation/Example.lean Co-authored-by: Ruben Van de Velde <[email protected]> --------- Co-authored-by: Ruben Van de Velde <[email protected]>
1 parent d5f9eb8 commit f9bca0d

File tree

8 files changed

+6
-20
lines changed

8 files changed

+6
-20
lines changed

FLT.lean

-1
Original file line numberDiff line numberDiff line change
@@ -27,7 +27,6 @@ import FLT.Mathlib.Algebra.Algebra.Hom
2727
import FLT.Mathlib.Algebra.Algebra.Pi
2828
import FLT.Mathlib.Algebra.Algebra.Tower
2929
import FLT.Mathlib.Algebra.BigOperators.Group.Finset.Basic
30-
import FLT.Mathlib.Algebra.Group.Subgroup.Defs
3130
import FLT.Mathlib.Algebra.Module.LinearMap.Defs
3231
import FLT.Mathlib.Algebra.Order.AbsoluteValue.Basic
3332
import FLT.Mathlib.Algebra.Order.Hom.Monoid

FLT/AutomorphicRepresentation/Example.lean

+1-1
Original file line numberDiff line numberDiff line change
@@ -650,7 +650,7 @@ lemma preserves_zsmul {G H : Type*} [Zero G] [Add G] [Neg G] [SMul ℕ G] [SubNe
650650
(neg : ∀ x, f (-x) = - f x)
651651
(z : ℤ) (g : G) :
652652
f (zsmulRec (· • ·) z g) = z • f g := by
653-
induction z with
653+
cases z with
654654
| ofNat n =>
655655
rw [zsmulRec, nsmul, Int.ofNat_eq_coe, natCast_zsmul]
656656
| negSucc n =>

FLT/DedekindDomain/FiniteAdeleRing/BaseChange.lean

+3-3
Original file line numberDiff line numberDiff line change
@@ -141,9 +141,9 @@ lemma intValuation_comap (hAB : Function.Injective (algebraMap A B))
141141
omit [IsIntegralClosure B A L] [FiniteDimensional K L] [Algebra.IsSeparable K L]
142142
[Module.Finite A B] in
143143
lemma valuation_comap (w : HeightOneSpectrum B) (x : K) :
144-
(comap A w).valuation x ^
144+
(comap A w).valuation K x ^
145145
(Ideal.ramificationIdx (algebraMap A B) (comap A w).asIdeal w.asIdeal) =
146-
w.valuation (algebraMap K L x) := by
146+
w.valuation L (algebraMap K L x) := by
147147
obtain ⟨x, y, hy, rfl⟩ := IsFractionRing.div_surjective (A := A) x
148148
simp [valuation, ← IsScalarTower.algebraMap_apply A K L, IsScalarTower.algebraMap_apply A B L,
149149
← intValuation_comap A B (algebraMap_injective_of_field_isFractionRing A B K L), div_pow]
@@ -177,7 +177,7 @@ lemma _root_.IsDedekindDomain.HeightOneSpectrum.adicValued.continuous_algebraMap
177177
refine ⟨a / m, fun x hx ↦ ?_⟩
178178
simp_rw [← valuation_comap A]
179179
calc
180-
(comap A w).valuation x ^ m < e (a / ↑m) ^ m := by gcongr; exacts [zero_le', hx]
180+
(comap A w).valuation K x ^ m < e (a / ↑m) ^ m := by gcongr; exacts [zero_le', hx]
181181
_ = e (m • (a / ↑m)) := by
182182
dsimp [e]
183183
norm_cast

FLT/HaarMeasure/DistribHaarChar/RealComplex.lean

+1-1
Original file line numberDiff line numberDiff line change
@@ -62,7 +62,7 @@ lemma distribHaarChar_complex (z : ℂˣ) : distribHaarChar ℂ z = ‖(z : ℂ)
6262
(f := (LinearMap.mul ℂ ℂ z⁻¹).restrictScalars ℝ) _ _ using 2
6363
· simpa [LinearMap.mul, LinearMap.mk₂, LinearMap.mk₂', LinearMap.mk₂'ₛₗ, Units.smul_def, eq_comm]
6464
using preimage_smul_inv z (Icc 0 1 ×ℂ Icc 0 1)
65-
· simp [key, ofReal_norm_eq_enorm, ← Complex.norm_eq_abs, ENNReal.ofReal_pow, zpow_ofNat]; rfl
65+
· simp [key, ofReal_norm_eq_enorm, ENNReal.ofReal_pow, zpow_ofNat]; rfl
6666
· simp [key, zpow_ofNat]
6767

6868
lemma Complex.volume_complex_smul (z : ℂ) (s : Set ℂ) : volume (z • s) = ‖z‖₊ ^ 2 * volume s := by

FLT/Mathlib/Algebra/Group/Subgroup/Defs.lean

-6
This file was deleted.

FLT/Mathlib/MeasureTheory/Group/Action.lean

-1
Original file line numberDiff line numberDiff line change
@@ -1,7 +1,6 @@
11
import Mathlib.MeasureTheory.Group.Action
22
import Mathlib.MeasureTheory.Group.Pointwise
33
import Mathlib.Topology.Algebra.InfiniteSum.ENNReal
4-
import FLT.Mathlib.Algebra.Group.Subgroup.Defs
54
import FLT.Mathlib.GroupTheory.Complement
65
import FLT.Mathlib.GroupTheory.Index
76

FLT/Mathlib/Topology/Constructions.lean

-6
Original file line numberDiff line numberDiff line change
@@ -6,9 +6,3 @@ theorem TopologicalSpace.prod_mono {α β : Type*} {σ₁ σ₂ : TopologicalSpa
66
@instTopologicalSpaceProd α β σ₁ τ₁ ≤ @instTopologicalSpaceProd α β σ₂ τ₂ :=
77
le_inf (inf_le_left.trans <| induced_mono hσ)
88
(inf_le_right.trans <| induced_mono hτ)
9-
10-
theorem DenseRange.piMap {ι : Type*} {X Y : ι → Type*} [∀ i, TopologicalSpace (Y i)]
11-
{f : (i : ι) → (X i) → (Y i)} (hf : ∀ i, DenseRange (f i)):
12-
DenseRange (Pi.map f) := by
13-
rw [DenseRange, Set.range_piMap]
14-
exact dense_pi Set.univ (fun i _ => hf i)

lake-manifest.json

+1-1
Original file line numberDiff line numberDiff line change
@@ -15,7 +15,7 @@
1515
"type": "git",
1616
"subDir": null,
1717
"scope": "",
18-
"rev": "2836c275479466837c2593377bb54ae9fafc41d2",
18+
"rev": "6d33eaf659620a8f914d9c9489dad0d27be88610",
1919
"name": "mathlib",
2020
"manifestFile": "lake-manifest.json",
2121
"inputRev": "master",

0 commit comments

Comments
 (0)