Skip to content

Commit

Permalink
Browse files Browse the repository at this point in the history
  • Loading branch information
alexjbest committed Nov 29, 2023
2 parents 18d9aa7 + 303420d commit c025b1c
Showing 1 changed file with 17 additions and 2 deletions.
19 changes: 17 additions & 2 deletions FltRegular/NumberTheory/Hilbert92.lean
Original file line number Diff line number Diff line change
Expand Up @@ -39,8 +39,23 @@ def systemOfUnits.IsFundamental [Module A G] (h : systemOfUnits p G σ r) :=
∀ s : systemOfUnits p G σ r, h.index ≤ s.index

namespace systemOfUnits
lemma existence' [Module A G] (S : systemOfUnits p G σ R) : ∃ S : systemOfUnits p G σ (R + 1), True := sorry
lemma existence (r) [Module A G] : ∃ S : systemOfUnits p G σ r, True := sorry

lemma existence0 [Module A G] : Nonempty (systemOfUnits p G σ 0) := by
refine ⟨⟨fun _ => 0, linearIndependent_empty_type⟩⟩

lemma existence' [Module A G] (S : systemOfUnits p G σ R) (hR : R < r) :
Nonempty (systemOfUnits p G σ (R + 1)) := sorry

lemma existence'' [Module A G] (hR : R ≤ r) : Nonempty (systemOfUnits p G σ R) := by
induction R with
| zero => exact existence0 p G σ
| succ n ih =>
obtain ⟨S⟩ := ih (le_trans (Nat.le_succ n) hR)
exact existence' p G σ S (lt_of_lt_of_le (Nat.lt.base n) hR)

lemma existence (r) [Module A G] : Nonempty (systemOfUnits p G σ r) := existence'' p G σ rfl.le


end systemOfUnits

noncomputable
Expand Down

0 comments on commit c025b1c

Please sign in to comment.