-
Notifications
You must be signed in to change notification settings - Fork 298
[Merged by Bors] - refactor(set_theory/game/pgame): rename and add theorems like -y ≤ -x ↔ x ≤ y
#14653
Conversation
src/set_theory/game/pgame.lean
Outdated
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⟩ |
There was a problem hiding this comment.
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
There was a problem hiding this comment.
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.
There was a problem hiding this comment.
Choose a reason for hiding this comment
The reason will be displayed to describe this comment to others. Learn more.
bors d+
Thanks!
✌️ vihdzp can now approve this pull request. To approve and merge a pull request, simply reply with |
bors r+ |
…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.
Pull request successfully merged into master. Build succeeded: |
-y ≤ -x ↔ x ≤ y
-y ≤ -x ↔ x ≤ y
For
*
inle
,lf
,lt
, we renameneg_*_iff : -y * -x ↔ x * y
toneg_*_neg_iff
, and add the theoremsneg_*_iff : -y * x ↔ x * -y
.We further add many missing corresponding theorems for equivalence and fuzziness.