Skip to content

Commit

Permalink
bump
Browse files Browse the repository at this point in the history
  • Loading branch information
riccardobrasca committed Dec 29, 2024
1 parent c0d3922 commit fbe1ae5
Show file tree
Hide file tree
Showing 2 changed files with 8 additions and 8 deletions.
8 changes: 4 additions & 4 deletions FltRegular/NumberTheory/Hilbert92.lean
Original file line number Diff line number Diff line change
Expand Up @@ -130,7 +130,7 @@ lemma lemma2 [Module A G] (S : systemOfUnits p G s) (hs : S.IsFundamental)
let a' := a.comapDomain (Fin.succAbove i) Fin.succAbove_right_injective.injOn
have hS' : S'.units ∘ Fin.succAbove i = S.units ∘ Fin.succAbove i := by
ext; simp only [Function.comp_apply, ne_eq, Fin.succAbove_ne, not_false_eq_true,
Function.update_noteq]
Function.update_of_ne]
have ha' :
Finsupp.linearCombination A (S'.units ∘ Fin.succAbove i) a' + S.units i = (1 - zeta p) • g := by
rw [hS', Finsupp.linearCombination_comp, LinearMap.comp_apply, Finsupp.lmapDomain_apply,
Expand Down Expand Up @@ -158,11 +158,11 @@ lemma lemma2 [Module A G] (S : systemOfUnits p G s) (hs : S.IsFundamental)
· rw [add_comm, ← eq_sub_iff_add_eq] at ha'
rw [← hij, ha']
apply sub_mem
· exact Submodule.smul_mem _ _ (Submodule.subset_span ⟨i, Function.update_same _ _ _⟩)
· exact Submodule.smul_mem _ _ (Submodule.subset_span ⟨i, Function.update_self _ _ _⟩)
· rw [← Finsupp.range_linearCombination, Finsupp.linearCombination_comp, LinearMap.comp_apply]
exact ⟨_, rfl⟩
· exact Submodule.subset_span ⟨j, Function.update_noteq (Ne.symm hij) _ _⟩
· refine ⟨g, Submodule.subset_span ⟨i, Function.update_same _ _ _⟩, ?_⟩
· exact Submodule.subset_span ⟨j, Function.update_of_ne (Ne.symm hij) _ _⟩
· refine ⟨g, Submodule.subset_span ⟨i, Function.update_self _ _ _⟩, ?_⟩
rw [← Finsupp.range_linearCombination]
rintro ⟨l, rfl⟩
letI := (Algebra.id A).toModule
Expand Down
8 changes: 4 additions & 4 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": "",
"rev": "fd52917a1ac853bcb73cd089ce43e6a4257c98e0",
"rev": "43d30441447b3b8da2ae24e2091751feb743640c",
"name": "«doc-gen4»",
"manifestFile": "lake-manifest.json",
"inputRev": "main",
Expand All @@ -15,7 +15,7 @@
"type": "git",
"subDir": null,
"scope": "",
"rev": "7edf946a4217aa3aa911290811204096e8464ada",
"rev": "75d7aea6c81efeb68701164edaaa9116f06b91ba",
"name": "checkdecls",
"manifestFile": "lake-manifest.json",
"inputRev": "master",
Expand All @@ -25,7 +25,7 @@
"type": "git",
"subDir": null,
"scope": "",
"rev": "d4736a1fb2613cc1c6eac9321e0471f744ff3551",
"rev": "58dc043d6bdac239bfbdcb8de5257893aac92baa",
"name": "mathlib",
"manifestFile": "lake-manifest.json",
"inputRev": null,
Expand Down Expand Up @@ -85,7 +85,7 @@
"type": "git",
"subDir": null,
"scope": "leanprover-community",
"rev": "d7caecce0d0f003fd5e9cce9a61f1dd6ba83142b",
"rev": "003ff459cdd85de551f4dcf95cdfeefe10f20531",
"name": "LeanSearchClient",
"manifestFile": "lake-manifest.json",
"inputRev": "main",
Expand Down

0 comments on commit fbe1ae5

Please sign in to comment.