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