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

feat(set_theory/game/pgame): define pgame.identical pgame.memₗ pgame.memᵣ #18515

Closed
wants to merge 22 commits into from

Conversation

FR-vdash-bot
Copy link
Collaborator

@FR-vdash-bot FR-vdash-bot commented Feb 28, 2023

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 as eq.

Zulip


Open in Gitpod

@FR-vdash-bot FR-vdash-bot added awaiting-review The author would like community review of the PR awaiting-CI The author would like to see what CI has to say before doing more work. labels Feb 28, 2023
@FR-vdash-bot FR-vdash-bot changed the title feat(set_theory/game/pgame): define pgame.identical feat(set_theory/game/pgame): define pgame.identical pgame.memₗ pgame.memᵣ Feb 28, 2023
@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 Mar 1, 2023
Copy link
Collaborator

@vihdzp vihdzp left a 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.

src/set_theory/game/basic.lean Show resolved Hide resolved
src/set_theory/game/pgame.lean Show resolved Hide resolved
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))) ∧
Copy link
Collaborator

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?

Copy link
Collaborator Author

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...

Copy link
Collaborator

Choose a reason for hiding this comment

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

Ah, me neither unfortunately.

src/set_theory/game/pgame.lean Outdated Show resolved Hide resolved
src/set_theory/game/basic.lean Show resolved Hide resolved
src/set_theory/game/pgame.lean Outdated Show resolved Hide resolved
Co-authored-by: Yaël Dillies <[email protected]>
Copy link
Collaborator

@vihdzp vihdzp left a 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.

src/set_theory/game/basic.lean Show resolved Hide resolved
src/set_theory/game/pgame.lean Outdated Show resolved Hide resolved
Co-authored-by: Yaël Dillies <[email protected]>
src/set_theory/game/basic.lean Outdated Show resolved Hide resolved
src/set_theory/game/pgame.lean Outdated Show resolved Hide resolved
src/set_theory/game/pgame.lean Outdated Show resolved Hide resolved
FR-vdash-bot and others added 2 commits March 30, 2023 21:36
Co-authored-by: Yaël Dillies <[email protected]>
@vihdzp
Copy link
Collaborator

vihdzp commented Apr 2, 2023

I've separated the forall_exists_rel bit into #18713.

@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
@kim-em
Copy link
Collaborator

kim-em commented Jul 27, 2023

I'm closing this as its been replaced by leanprover-community/mathlib4#5901

@kim-em kim-em closed this Jul 27, 2023
@YaelDillies YaelDillies deleted the FR_game_identical branch August 28, 2023 13:26
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 not-too-late This PR was ready at the point mathlib3 was frozen: we will try to merge it and port it to mathlib4
Projects
None yet
Development

Successfully merging this pull request may close these issues.

5 participants