Commit 2023-11-03 16:13 2e15c5a0

View on Github โ†’

feat: use Minkowski's theorem to prove the existence of algebraic integers of small norm (#8128) We define the convex body convexBodySum and prove the following

theorem exists_ne_zero_mem_ringOfIntegers_of_norm_le {B : โ„}
     (h : (minkowskiBound K) < volume (convexBodySum K B)) :
     โˆƒ (a : ๐“ž K), a โ‰  0 โˆง |Algebra.norm โ„š (a:K)| โ‰ค ((finrank โ„š K : โ„)โปยน * B) ^ (finrank โ„š K) 

Computation of the volume (convexBodySum K B)) and applications of the result are coming in a following PR.

Estimated changes