Skip to content

Commit

Permalink
Fix comment typo from the port; ought to regenerate the blueprint.
Browse files Browse the repository at this point in the history
  • Loading branch information
grunweg committed Feb 6, 2024
1 parent 5c609a5 commit 5487c14
Show file tree
Hide file tree
Showing 2 changed files with 2 additions and 2 deletions.
2 changes: 1 addition & 1 deletion SphereEversion/Local/AmpleSet.lean
Original file line number Diff line number Diff line change
Expand Up @@ -67,7 +67,7 @@ theorem AmpleSet.preimage {s : Set F} (h : AmpleSet s) (L : E ≃L[ℝ] F) : Amp
open scoped Pointwise

/-- Translating a ample set is ample.
We basically mimic `ample_set.image`. We could prove the common generalization using
We basically mimic `AmpleSet.image`. We could prove the common generalization using
continuous affine equivalences -/
theorem AmpleSet.vadd [ContinuousAdd E] {s : Set E} (h : AmpleSet s) {y : E} :
AmpleSet (y +ᵥ s) := by
Expand Down
2 changes: 1 addition & 1 deletion blueprint/src/local_convex_integration.tex
Original file line number Diff line number Diff line change
Expand Up @@ -319,7 +319,7 @@ \section{Ample differential relations}
\begin{definition}
\label{def:ample_subset}
\leanok
\lean{ample_set}
\lean{AmpleSet}
A subset $Ω$ of a real vector space $E$ is ample if the convex
hull of each connected component of $Ω$ is the whole $E$.
\end{definition}
Expand Down

0 comments on commit 5487c14

Please sign in to comment.