Skip to content

Commit

Permalink
chore(Partition): tinygolf
Browse files Browse the repository at this point in the history
  • Loading branch information
grunweg committed Apr 17, 2024
1 parent 57b10af commit fb10b9a
Showing 1 changed file with 1 addition and 2 deletions.
3 changes: 1 addition & 2 deletions SphereEversion/ToMathlib/Partition.lean
Original file line number Diff line number Diff line change
Expand Up @@ -53,8 +53,7 @@ theorem germ_combine_mem (φ : ι → M → F) (hx : x ∈ interior s := by simp
rw [this]
refine sum_mem_reallyConvexHull ?_ (ρ.sum_germ hx) (fun i hi ↦ mem_image_of_mem _ hi)
· intro i _
filter_upwards
apply ρ.nonneg
filter_upwards using fun a ↦ ρ.nonneg i a

end SmoothPartitionOfUnity

Expand Down

0 comments on commit fb10b9a

Please sign in to comment.