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

[Merged by Bors] - refactor(set_theory/game/pgame): rename and add theorems like -y ≤ -x ↔ x ≤ y #14653

Closed
wants to merge 7 commits into from

Conversation

vihdzp
Copy link
Collaborator

@vihdzp vihdzp commented Jun 9, 2022

For * in le, lf, lt, we rename neg_*_iff : -y * -x ↔ x * y to neg_*_neg_iff, and add the theorems neg_*_iff : -y * x ↔ x * -y.

We further add many missing corresponding theorems for equivalence and fuzziness.


Open in Gitpod

@vihdzp vihdzp added the awaiting-review The author would like community review of the PR label Jun 9, 2022
src/set_theory/game/pgame.lean Outdated Show resolved Hide resolved
by rw [←neg_fuzzy_iff, pgame.neg_zero]

theorem neg_congr {x y : pgame} (h : x ≈ y) : -x ≈ -y :=
⟨neg_le_neg_iff.2 h.2, neg_le_neg_iff.2 h.1⟩
Copy link
Member

Choose a reason for hiding this comment

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

This is now just neg_equiv_neg_iff.2 h, isn't it?

Also, this might be better named equiv.neg for dot notation

Copy link
Collaborator Author

@vihdzp vihdzp Jun 10, 2022

Choose a reason for hiding this comment

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

I'll just remove this theorem for now. If we decide in the future that the forward directions of these lemmas deserve names, I'll be sure to give them dot notation.

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+

Thanks!

@bors
Copy link

bors bot commented Jun 10, 2022

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

@leanprover-community-bot-assistant leanprover-community-bot-assistant added delegated The PR author may merge after reviewing final suggestions. and removed awaiting-review The author would like community review of the PR labels Jun 10, 2022
@vihdzp vihdzp added the awaiting-CI The author would like to see what CI has to say before doing more work. label Jun 10, 2022
@github-actions github-actions bot removed the awaiting-CI The author would like to see what CI has to say before doing more work. label Jun 10, 2022
@vihdzp
Copy link
Collaborator Author

vihdzp commented Jun 10, 2022

bors r+

bors bot pushed a commit that referenced this pull request Jun 10, 2022
…x ↔ x ≤ y` (#14653)

For `*` in `le`, `lf`, `lt`, we rename `neg_*_iff : -y * -x ↔ x * y` to `neg_*_neg_iff`, and add the theorems `neg_*_iff : -y * x ↔ x * -y`.

We further add many missing corresponding theorems for equivalence and fuzziness.
@bors
Copy link

bors bot commented Jun 10, 2022

Pull request successfully merged into master.

Build succeeded:

@bors bors bot changed the title refactor(set_theory/game/pgame): rename and add theorems like -y ≤ -x ↔ x ≤ y [Merged by Bors] - refactor(set_theory/game/pgame): rename and add theorems like -y ≤ -x ↔ x ≤ y Jun 10, 2022
@bors bors bot closed this Jun 10, 2022
@bors bors bot deleted the neg_lemmas_pgame branch June 10, 2022 10:43
Sign up for free to subscribe to this conversation on GitHub. Already have an account? Sign in.
Labels
delegated The PR author may merge after reviewing final suggestions.
Projects
None yet
Development

Successfully merging this pull request may close these issues.

4 participants