-
Notifications
You must be signed in to change notification settings - Fork 298
feat(set_theory/game/pgame): define pgame.identical
pgame.memₗ
pgame.memᵣ
#18515
Conversation
pgame.identical
pgame.identical
pgame.memₗ
pgame.memᵣ
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 was something that had been irking me for the longest time, thank you! Here's some initial remarks.
every right move of `x` is identical to some right move of `y`, and vice versa. -/ | ||
def identical : Π (x y : pgame), Prop | ||
| (mk _ _ xL xR) (mk _ _ yL yR) := | ||
((∀ i, ∃ j, identical (xL i) (yL j)) ∧ (∀ j, ∃ i, identical (xL i) (yL j))) ∧ |
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.
Can you use forall_exists_rel
in this definition?
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'm not sure how to show it is well-founded recursion to Lean...
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.
Ah, me neither unfortunately.
Co-authored-by: Yaël Dillies <[email protected]>
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.
Checking again, looks all good.
Co-authored-by: Yaël Dillies <[email protected]>
Co-authored-by: Yaël Dillies <[email protected]>
I've separated the |
I'm closing this as its been replaced by leanprover-community/mathlib4#5901 |
This PR is the first step to remove
pgame.relabelling
(which is only for implementing things in lean and not real identity) and define games with identity aseq
.Zulip