Skip to content

Commit

Permalink
fix spanA_eq_spanZ
Browse files Browse the repository at this point in the history
  • Loading branch information
erdOne committed Nov 30, 2023
1 parent fd28cac commit d208e82
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion FltRegular/NumberTheory/SystemOfUnits.lean
Original file line number Diff line number Diff line change
Expand Up @@ -126,7 +126,7 @@ lemma spanA_eq_spanZ [Module A G] {R : ℕ} (f : Fin R → G) :
· intro z w hz hw
exact Submodule.add_mem _ hz hw
· intro a _ hx
exact mem_spanS p G a f hx
exact mem_spanS p hp G _ f hx

lemma ex_not_mem [Module A G] {R : ℕ} (S : systemOfUnits p G R) (hR : R < r) :
∃ g, ∀ (k : ℤ), ¬(k • g ∈ Submodule.span A (Set.range S.units)) := by
Expand Down

0 comments on commit d208e82

Please sign in to comment.