Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit 1e9b3df

Browse files
committed
refactor(geometry/euclidean/basic): rename cospherical_subset (#16947)
Rename `cospherical_subset` to `cospherical.subset` to allow use of dot notation.
1 parent a08db7e commit 1e9b3df

File tree

1 file changed

+2
-2
lines changed

1 file changed

+2
-2
lines changed

src/geometry/euclidean/basic.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -757,7 +757,7 @@ lemma sphere.cospherical (s : sphere P) : cospherical (s : set P) :=
757757
cospherical_iff_exists_sphere.2 ⟨s, set.subset.rfl⟩
758758

759759
/-- A subset of a cospherical set is cospherical. -/
760-
lemma cospherical_subset {ps₁ ps₂ : set P} (hs : ps₁ ⊆ ps₂) (hc : cospherical ps₂) :
760+
lemma cospherical.subset {ps₁ ps₂ : set P} (hs : ps₁ ⊆ ps₂) (hc : cospherical ps₂) :
761761
cospherical ps₁ :=
762762
begin
763763
rcases hc with ⟨c, r, hcr⟩,
@@ -878,7 +878,7 @@ structure concyclic (ps : set P) : Prop :=
878878

879879
/-- A subset of a concyclic set is concyclic. -/
880880
lemma concyclic.subset {ps₁ ps₂ : set P} (hs : ps₁ ⊆ ps₂) (h : concyclic ps₂) : concyclic ps₁ :=
881-
cospherical_subset hs h.1, h.2.subset hs⟩
881+
⟨h.1.subset hs, h.2.subset hs⟩
882882

883883
/-- The empty set is concyclic. -/
884884
lemma concyclic_empty : concyclic (∅ : set P) :=

0 commit comments

Comments
 (0)