Commit 2023-09-08 11:01 248b0091

View on Github →

feat: compute the integral of sqrt (1 - x ^ 2) (#6905) We prove

theorem integral_sqrt_one_sub_sq : ∫ x in (-1 : ℝ)..1, sqrt (1 - x ^ 2) = π / 2

which will in turn be used to compute the area of the disc and then the volume of the unit complex ball in #6907

Estimated changes