Zulip Chat Archive
Stream: new members
Topic: ball
BANGJI HU (Oct 04 2024 at 14:12):
hi,everyone my problem is how to proove An object with a circle on any slice is a ball,and i d like hint,
BANGJI HU (Oct 04 2024 at 14:13):
import Mathlib.Geometry.Euclidean.Basic
def is_sphere (S : set ℝ³) : Prop :=
∃ (c : ℝ³) (r : ℝ), S = {x : ℝ³ | ∥x - c∥ = r}
def is_circle (C : set ℝ³) : Prop :=
∃ (p : plane ℝ³) (c : ℝ³) (r : ℝ), C = {x : ℝ³ | x ∈ p ∧ ∥x - c∥ = r}
def all_sections_are_circles (S : set ℝ³) : Prop :=
∀ (p : plane ℝ³), is_circle (S ∩ p.to_set)
theorem sections_are_circles_iff_sphere (S : set ℝ³) :
all_sections_are_circles S ↔ is_sphere S :=
Damiano Testa (Oct 04 2024 at 14:18):
Opening this, I get expected token
.
Last updated: May 02 2025 at 03:31 UTC