Skip to content
New issue

Have a question about this project? Sign up for a free GitHub account to open an issue and contact its maintainers and the community.

By clicking “Sign up for GitHub”, you agree to our terms of service and privacy statement. We’ll occasionally send you account related emails.

Already on GitHub? Sign in to your account

[Merged by Bors] - feat(analysis/seminorm): semilattice_sup on seminorms and lemmas about ball #11329

Closed
wants to merge 52 commits into from

Conversation

mcdoll
Copy link
Member

@mcdoll mcdoll commented Jan 9, 2022

Define bot and the the binary sup on seminorms, and some lemmas about the supremum of a finite number of seminorms.
Shows that the unit ball of the supremum is given by the intersection of the unit balls.

Co-authored-by: Eric Wieser wieser.eric@gmail.com


Open in Gitpod

@mcdoll
Copy link
Member Author

mcdoll commented Jan 9, 2022

There might be quite some room for golfing and I don't know whether there is an easier solution to deal with nnreal.

@mcdoll mcdoll added the awaiting-CI The author would like to see what CI has to say before doing more work. label Jan 9, 2022
@eric-wieser
Copy link
Member

eric-wieser commented Jan 9, 2022

Can you instead provide a semilattice_sup and order_bot instance on seminorm? That way finset.sup is the definition in this PR.

@eric-wieser eric-wieser added the awaiting-author A reviewer has asked the author a question or requested changes label Jan 9, 2022
@eric-wieser
Copy link
Member

eric-wieser commented Jan 9, 2022

A template to get you started:

-- this belongs immediately after the `has_coe_to_fun` instance
lemma coe_injective : @function.injective (seminorm 𝕜 E) (E → ℝ) coe_fn
| ⟨x, _, _⟩ ⟨y, _, _⟩ rfl := rfl

instance : has_sup (seminorm 𝕜 E) :=
{ sup := λ x y,
  { to_fun := x ⊔ y,
    triangle' := sorry,
    smul' := sorry }}

@[simp] lemma coe_sup (x y : seminorm 𝕜 E) : ⇑(x ⊔ y) = x ⊔ y := rfl

instance : semilattice_sup (seminorm 𝕜 E) :=
function.injective.semilattice_sup _ coe_injective coe_sup

instance : order_bot (seminorm 𝕜 E) :=
{ bot :=
  { to_fun := 0,
    triangle' := λ x y, by simp,
    smul' := λ k x, by simp },
  bot_le := nonneg }

@[simp] lemma coe_bot : ⇑(⊥ : seminorm 𝕜 E) = 0 := rfl

@mcdoll
Copy link
Member Author

mcdoll commented Jan 9, 2022

ah thanks, I will try that.

@eric-wieser
Copy link
Member

With that in place, the new definition is just:

def seminorm_sup_finset (p : ι → seminorm 𝕜 E) (ι' : finset ι) : seminorm 𝕜 E :=
  ι'.sup p

which of course doesn't need to exist any more.

@mcdoll
Copy link
Member Author

mcdoll commented Jan 9, 2022

@eric-wieser it works perfectly. I need two lemmas that have nothing to do with seminorms: sup_eq_sup for sup-semilattices and mul_sup for the reals (was written by @user7230724 ), should I make separate PRs for them or is it ok to have them in this PR?

@eric-wieser
Copy link
Member

Push them to this PR for now, then we can discuss moving them

@mcdoll
Copy link
Member Author

mcdoll commented Jan 9, 2022

I don't really understand how to unfold ι'.sup p, I tried to apply in l. 527 finset.sup_induction (which doesn't seems to be the correction thing in the first place), but I failed.

mcdoll and others added 3 commits January 9, 2022 22:10
Co-authored-by: Eric Wieser <wieser.eric@gmail.com>
mcdoll and others added 3 commits January 14, 2022 13:37
Co-authored-by: Yaël Dillies <yael.dillies@gmail.com>
@eric-wieser eric-wieser changed the title feat(analysis/seminorm): Add finite supremum of seminorms feat(analysis/seminorm): semilattice_sup on seminorms and lemmas about ball Jan 14, 2022
Copy link
Member

@eric-wieser eric-wieser left a comment

Choose a reason for hiding this comment

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

bors d+

@bors
Copy link

bors bot commented Jan 14, 2022

✌️ mcdoll can now approve this pull request. To approve and merge a pull request, simply reply with bors r+. More detailed instructions are available here.

mcdoll and others added 3 commits January 14, 2022 14:29
Co-authored-by: Eric Wieser <wieser.eric@gmail.com>
Co-authored-by: Eric Wieser <wieser.eric@gmail.com>
mcdoll and others added 2 commits January 14, 2022 16:31
Co-authored-by: Eric Wieser <wieser.eric@gmail.com>
@mcdoll
Copy link
Member Author

mcdoll commented Jan 14, 2022

bors merge

bors bot pushed a commit that referenced this pull request Jan 14, 2022
…out `ball` (#11329)

Define `bot` and the the binary `sup` on seminorms, and some lemmas about the supremum of a finite number of seminorms.
Shows that the unit ball of the supremum is given by the intersection of the unit balls.


Co-authored-by: Eric Wieser <wieser.eric@gmail.com>
@bors
Copy link

bors bot commented Jan 14, 2022

Pull request successfully merged into master.

Build succeeded:

@bors bors bot changed the title feat(analysis/seminorm): semilattice_sup on seminorms and lemmas about ball [Merged by Bors] - feat(analysis/seminorm): semilattice_sup on seminorms and lemmas about ball Jan 14, 2022
@bors bors bot closed this Jan 14, 2022
@bors bors bot deleted the mcdoll/seminorm_sup branch January 14, 2022 19:02
bors bot pushed a commit that referenced this pull request Mar 12, 2022
…12624)

Move `balanced`, `absorbs`, `absorbent` to a new file.

For `analysis.seminorm`, I'm crediting
* Jean for #4827
* myself for
  * #9097
  * #11487
* Moritz for
  * #11329
  * #11414
  * #11477

For `analysis.locally_convex.basic`, I'm crediting
* Jean for #4827
* Bhavik for
  * #7358
  * #9097
* myself for
  * #9097
  * #10999
  * #11487
laurentbartholdi pushed a commit that referenced this pull request Mar 17, 2022
…12624)

Move `balanced`, `absorbs`, `absorbent` to a new file.

For `analysis.seminorm`, I'm crediting
* Jean for #4827
* myself for
  * #9097
  * #11487
* Moritz for
  * #11329
  * #11414
  * #11477

For `analysis.locally_convex.basic`, I'm crediting
* Jean for #4827
* Bhavik for
  * #7358
  * #9097
* myself for
  * #9097
  * #10999
  * #11487
Sign up for free to join this conversation on GitHub. Already have an account? Sign in to comment
Labels
delegated The PR author may merge after reviewing final suggestions.
Projects
None yet
Development

Successfully merging this pull request may close these issues.

None yet

6 participants