Skip to content

Commit

Permalink
bump
Browse files Browse the repository at this point in the history
  • Loading branch information
riccardobrasca committed Nov 23, 2024
1 parent 8973e0d commit 438ada3
Show file tree
Hide file tree
Showing 2 changed files with 5 additions and 17 deletions.
18 changes: 3 additions & 15 deletions FltRegular/NumberTheory/Hilbert92.lean
Original file line number Diff line number Diff line change
Expand Up @@ -92,20 +92,6 @@ lemma LinearIndependent.update {ι} [DecidableEq ι] {R} [CommRing R] [Module R
ext j
exact hσ _ ((mul_comm _ _).trans (hl' j))

@[to_additive]
lemma Subgroup.index_mono {G : Type*} [Group G] {H₁ H₂ : Subgroup G} (h : H₁ < H₂)
[h₁ : Fintype (G ⧸ H₁)] :
H₂.index < H₁.index := by
rcases eq_or_ne H₂.index 0 with hn | hn
· rw [hn, index_eq_card, Nat.card_eq_fintype_card]
exact Fintype.card_pos
apply lt_of_le_of_ne
refine Nat.le_of_dvd (by rw [index_eq_card, Nat.card_eq_fintype_card]; apply Fintype.card_pos)
<| Subgroup.index_dvd_of_le h.le
have := fintypeOfIndexNeZero hn
rw [←mul_one H₂.index, ←relindex_mul_index h.le, mul_comm, Ne, eq_comm]
simp [-one_mul, -Nat.one_mul, hn, h.not_le]

namespace systemOfUnits.IsFundamental

variable {H : Type*} [CommGroup H] [Fintype H]
Expand Down Expand Up @@ -160,7 +146,9 @@ lemma lemma2 [Module A G] (S : systemOfUnits p G s) (hs : S.IsFundamental)
Finsupp.comapDomain_apply]
letI := S'.isMaximal p hp G hf
suffices Submodule.span A (Set.range S.units) < Submodule.span A (Set.range S'.units) by
exact (hs.maximal' _ _ _ S').not_lt (AddSubgroup.index_mono (h₁ := S.isMaximal _ hp _ hf) this)
have : (Submodule.span A (Set.range S.units)).toAddSubgroup.FiniteIndex :=
⟨AddSubgroup.index_ne_zero_of_finite (hH := (S.isMaximal _ hp _ hf).finite)⟩
exact (hs.maximal' _ _ _ S').not_lt <| AddSubgroup.index_strictAnti ‹_›
rw [SetLike.lt_iff_le_and_exists]
constructor
· rw [Submodule.span_le]
Expand Down
4 changes: 2 additions & 2 deletions lake-manifest.json
Original file line number Diff line number Diff line change
Expand Up @@ -5,7 +5,7 @@
"type": "git",
"subDir": null,
"scope": "leanprover-community",
"rev": "a822446d61ad7e7f5e843365c7041c326553050a",
"rev": "8b52587ff32e2e443cce6109b5305341289339e7",
"name": "batteries",
"manifestFile": "lake-manifest.json",
"inputRev": "main",
Expand Down Expand Up @@ -85,7 +85,7 @@
"type": "git",
"subDir": null,
"scope": "",
"rev": "840e02ce2768e06de7ced0a624444746590e9d99",
"rev": "ff064a56e58e8ceb1c0a3febd60e701a1cf408fe",
"name": "mathlib",
"manifestFile": "lake-manifest.json",
"inputRev": null,
Expand Down

0 comments on commit 438ada3

Please sign in to comment.