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

feat(analysic/convex): add lemmas and defs about low-dimensional simplices #19101

Closed
wants to merge 3 commits into from

Conversation

urkud
Copy link
Member

@urkud urkud commented May 26, 2023

Motivated about a homeomorph statemnt from Shamrock-Frost/BrouwerFixedPoint

Co-authored-by: @Shamrock-Frost


Should lemmas about set equalities be simp? Or std_simplex should
be the normal form no matter what?

Open in Gitpod

@github-actions github-actions bot added the modifies-synchronized-file This PR touches a files that has already been ported to mathlib4, and may need a synchronization PR. label May 26, 2023
@urkud urkud added awaiting-review The author would like community review of the PR t-topology Topological spaces, uniform spaces, metric spaces, filters t-analysis Analysis (normed *, calculus) and removed modifies-synchronized-file This PR touches a files that has already been ported to mathlib4, and may need a synchronization PR. labels May 26, 2023

lemma ite_eq_mem_std_simplex (i : ι) : (λ j, ite (i = j) (1:𝕜) 0) ∈ std_simplex 𝕜 ι :=
⟨λ j, by simp only; split_ifs; norm_num, by rw [finset.sum_ite_eq, if_pos (finset.mem_univ _)]⟩

lemma single_mem_std_simplex (i : ι) : pi.single i 1 ∈ std_simplex 𝕜 ι :=
Copy link
Member

Choose a reason for hiding this comment

The reason will be displayed to describe this comment to others. Learn more.

I think this is missing a DecidableEq?

Copy link
Member Author

Choose a reason for hiding this comment

The reason will be displayed to describe this comment to others. Learn more.

There is a decidable_eq variable a few lines above.

@eric-wieser eric-wieser added awaiting-author A reviewer has asked the author a question or requested changes and removed awaiting-review The author would like community review of the PR labels May 28, 2023
@urkud urkud added the modifies-synchronized-file This PR touches a files that has already been ported to mathlib4, and may need a synchronization PR. label Jun 21, 2023
@urkud urkud added awaiting-review The author would like community review of the PR and removed awaiting-author A reviewer has asked the author a question or requested changes labels Jun 21, 2023
@urkud urkud requested a review from eric-wieser June 21, 2023 03:53
@eric-wieser eric-wieser added the not-too-late This PR was ready at the point mathlib3 was frozen: we will try to merge it and port it to mathlib4 label Jul 15, 2023
@urkud
Copy link
Member Author

urkud commented Jul 16, 2023

I'm going to port it using oneshot.

@urkud urkud added too-late This PR was ready too late for inclusion in mathlib3 and removed not-too-late This PR was ready at the point mathlib3 was frozen: we will try to merge it and port it to mathlib4 labels Jul 16, 2023
@urkud
Copy link
Member Author

urkud commented Feb 7, 2024

Forward-ported as leanprover-community/mathlib4#10325

@urkud urkud closed this Feb 7, 2024
@urkud urkud deleted the YK-std-simpl branch February 7, 2024 06:41
mathlib-bors bot pushed a commit to leanprover-community/mathlib4 that referenced this pull request Feb 8, 2024
atarnoam pushed a commit to leanprover-community/mathlib4 that referenced this pull request Feb 9, 2024
Sign up for free to subscribe to this conversation on GitHub. Already have an account? Sign in.
Labels
awaiting-review The author would like community review of the PR modifies-synchronized-file This PR touches a files that has already been ported to mathlib4, and may need a synchronization PR. t-analysis Analysis (normed *, calculus) t-topology Topological spaces, uniform spaces, metric spaces, filters too-late This PR was ready too late for inclusion in mathlib3
Projects
None yet
Development

Successfully merging this pull request may close these issues.

2 participants