Documentation

Mathlib.SetTheory.Game.PGame

Combinatorial (pre-)games. #

The basic theory of combinatorial games, following Conway's book On Numbers and Games. We construct "pregames", define an ordering and arithmetic operations on them, then show that the operations descend to "games", defined via the equivalence relation p ≈ q ↔ p ≤ q ∧ q ≤ p.

The surreal numbers will be built as a quotient of a subtype of pregames.

A pregame (SetTheory.PGame below) is axiomatised via an inductive type, whose sole constructor takes two types (thought of as indexing the possible moves for the players Left and Right), and a pair of functions out of these types to SetTheory.PGame (thought of as describing the resulting game after making a move).

Combinatorial games themselves, as a quotient of pregames, are constructed in Game.lean.

Conway induction #

By construction, the induction principle for pregames is exactly "Conway induction". That is, to prove some predicate SetTheory.PGame → Prop holds for all pregames, it suffices to prove that for every pregame g, if the predicate holds for every game resulting from making a move, then it also holds for g.

While it is often convenient to work "by induction" on pregames, in some situations this becomes awkward, so we also define accessor functions SetTheory.PGame.LeftMoves, SetTheory.PGame.RightMoves, SetTheory.PGame.moveLeft and SetTheory.PGame.moveRight. There is a relation PGame.Subsequent p q, saying that p can be reached by playing some non-empty sequence of moves starting from q, an instance WellFounded Subsequent, and a local tactic pgame_wf_tac which is helpful for discharging proof obligations in inductive proofs relying on this relation.

Order properties #

Pregames have both a and a < relation, satisfying the usual properties of a Preorder. The relation 0 < x means that x can always be won by Left, while 0 ≤ x means that x can be won by Left as the second player.

It turns out to be quite convenient to define various relations on top of these. We define the "less or fuzzy" relation x ⧏ y as ¬ y ≤ x, the equivalence relation x ≈ y as x ≤ y ∧ y ≤ x, and the fuzzy relation x ‖ y as x ⧏ y ∧ y ⧏ x. If 0 ⧏ x, then x can be won by Left as the first player. If x ≈ 0, then x can be won by the second player. If x ‖ 0, then x can be won by the first player.

Statements like zero_le_lf, zero_lf_le, etc. unfold these definitions. The theorems le_def and lf_def give a recursive characterisation of each relation in terms of themselves two moves later. The theorems zero_le, zero_lf, etc. also take into account that 0 has no moves.

Later, games will be defined as the quotient by the relation; that is to say, the Antisymmetrization of SetTheory.PGame.

Algebraic structures #

We next turn to defining the operations necessary to make games into a commutative additive group. Addition is defined for $x = {xL | xR}$ and $y = {yL | yR}$ by $x + y = {xL + y, x + yL | xR + y, x + yR}$. Negation is defined by ${xL | xR} = {-xR | -xL}$.

The order structures interact in the expected way with addition, so we have

theorem le_iff_sub_nonneg {x y : PGame} : x ≤ y ↔ 0 ≤ y - x := sorry
theorem lt_iff_sub_pos {x y : PGame} : x < y ↔ 0 < y - x := sorry

We show that these operations respect the equivalence relation, and hence descend to games. At the level of games, these operations satisfy all the laws of a commutative group. To prove the necessary equivalence relations at the level of pregames, we introduce the notion of a Relabelling of a game, and show, for example, that there is a relabelling between x + (y + z) and (x + y) + z.

Future work #

References #

The material here is all drawn from

An interested reader may like to formalise some of the material from

Pre-game moves #

inductive SetTheory.PGame :
Type (u + 1)

The type of pre-games, before we have quotiented by equivalence (PGame.Setoid). In ZFC, a combinatorial game is constructed from two sets of combinatorial games that have been constructed at an earlier stage. To do this in type theory, we say that a pre-game is built inductively from two families of pre-games indexed over any type in Type u. The resulting type PGame.{u} lives in Type (u+1), reflecting that it is a proper class in ZFC.

Instances For

    The indexing type for allowable moves by Left.

    Equations
    Instances For

      The indexing type for allowable moves by Right.

      Equations
      Instances For

        The new game after Left makes an allowed move.

        Equations
        Instances For

          The new game after Right makes an allowed move.

          Equations
          Instances For
            @[simp]
            theorem SetTheory.PGame.leftMoves_mk {xl : Type u_1} {xr : Type u_1} {xL : xlSetTheory.PGame} {xR : xrSetTheory.PGame} :
            @[simp]
            theorem SetTheory.PGame.moveLeft_mk {xl : Type u_1} {xr : Type u_1} {xL : xlSetTheory.PGame} {xR : xrSetTheory.PGame} :
            @[simp]
            theorem SetTheory.PGame.rightMoves_mk {xl : Type u_1} {xr : Type u_1} {xL : xlSetTheory.PGame} {xR : xrSetTheory.PGame} :
            @[simp]
            theorem SetTheory.PGame.moveRight_mk {xl : Type u_1} {xr : Type u_1} {xL : xlSetTheory.PGame} {xR : xrSetTheory.PGame} :

            Construct a pre-game from list of pre-games describing the available moves for Left and Right.

            Equations
            • One or more equations did not get rendered due to their size.
            Instances For

              Converts a number into a left move for ofLists.

              Equations
              • SetTheory.PGame.toOfListsLeftMoves = ((Equiv.cast ).trans Equiv.ulift).symm
              Instances For

                Converts a number into a right move for ofLists.

                Equations
                • SetTheory.PGame.toOfListsRightMoves = ((Equiv.cast ).trans Equiv.ulift).symm
                Instances For

                  A variant of PGame.recOn expressed in terms of PGame.moveLeft and PGame.moveRight.

                  Both this and PGame.recOn describe Conway induction on games.

                  Equations
                  Instances For

                    IsOption x y means that x is either a left or right option for y.

                    Instances For
                      theorem SetTheory.PGame.IsOption.mk_left {xl : Type u} {xr : Type u} (xL : xlSetTheory.PGame) (xR : xrSetTheory.PGame) (i : xl) :
                      theorem SetTheory.PGame.IsOption.mk_right {xl : Type u} {xr : Type u} (xL : xlSetTheory.PGame) (xR : xrSetTheory.PGame) (i : xr) :

                      Subsequent x y says that x can be obtained by playing some nonempty sequence of moves from y. It is the transitive closure of IsOption.

                      Equations
                      Instances For
                        @[simp]
                        theorem SetTheory.PGame.Subsequent.mk_left {xl : Type u_1} {xr : Type u_1} (xL : xlSetTheory.PGame) (xR : xrSetTheory.PGame) (i : xl) :
                        @[simp]
                        theorem SetTheory.PGame.Subsequent.mk_right {xl : Type u_1} {xr : Type u_1} (xL : xlSetTheory.PGame) (xR : xrSetTheory.PGame) (j : xr) :

                        Discharges proof obligations of the form Subsequent .. arising in termination proofs of definitions using well-founded recursion on PGame.

                        Equations
                        Instances For
                          @[simp]
                          theorem SetTheory.PGame.Subsequent.mk_right' {xl : Type u_1} {xr : Type u_1} (xL : xlSetTheory.PGame) (xR : xrSetTheory.PGame) (j : SetTheory.PGame.RightMoves (SetTheory.PGame.mk xl xr xL xR)) :
                          @[simp]
                          @[simp]
                          @[simp]

                          Basic pre-games #

                          The pre-game Zero is defined by 0 = { | }.

                          Equations

                          The pre-game One is defined by 1 = { 0 | }.

                          Equations

                          Pre-game order relations #

                          The less or equal relation on pre-games.

                          If 0 ≤ x, then Left can win x as the second player.

                          Equations
                          • One or more equations did not get rendered due to their size.

                          The less or fuzzy relation on pre-games.

                          If 0 ⧏ x, then Left can win x as the first player.

                          Equations
                          Instances For

                            The less or fuzzy relation on pre-games.

                            If 0 ⧏ x, then Left can win x as the first player.

                            Equations
                            • One or more equations did not get rendered due to their size.
                            Instances For

                              Definition of x ≤ y on pre-games, in terms of .

                              The ordering here is chosen so that And.left refer to moves by Left, and And.right refer to moves by Right.

                              @[simp]
                              theorem SetTheory.PGame.mk_le_mk {xl : Type u_1} {xr : Type u_1} {xL : xlSetTheory.PGame} {xR : xrSetTheory.PGame} {yl : Type u_1} {yr : Type u_1} {yL : ylSetTheory.PGame} {yR : yrSetTheory.PGame} :
                              SetTheory.PGame.mk xl xr xL xR SetTheory.PGame.mk yl yr yL yR (∀ (i : xl), SetTheory.PGame.LF (xL i) (SetTheory.PGame.mk yl yr yL yR)) ∀ (j : yr), SetTheory.PGame.LF (SetTheory.PGame.mk xl xr xL xR) (yR j)

                              Definition of x ≤ y on pre-games built using the constructor.

                              Definition of x ⧏ y on pre-games, in terms of .

                              The ordering here is chosen so that or.inl refer to moves by Left, and or.inr refer to moves by Right.

                              @[simp]
                              theorem SetTheory.PGame.mk_lf_mk {xl : Type u_1} {xr : Type u_1} {xL : xlSetTheory.PGame} {xR : xrSetTheory.PGame} {yl : Type u_1} {yr : Type u_1} {yL : ylSetTheory.PGame} {yR : yrSetTheory.PGame} :
                              SetTheory.PGame.LF (SetTheory.PGame.mk xl xr xL xR) (SetTheory.PGame.mk yl yr yL yR) (∃ (i : yl), SetTheory.PGame.mk xl xr xL xR yL i) ∃ (j : xr), xR j SetTheory.PGame.mk yl yr yL yR

                              Definition of x ⧏ y on pre-games built using the constructor.

                              theorem SetTheory.PGame.lf_of_le_mk {xl : Type u_1} {xr : Type u_1} {xL : xlSetTheory.PGame} {xR : xrSetTheory.PGame} {y : SetTheory.PGame} :
                              SetTheory.PGame.mk xl xr xL xR y∀ (i : xl), SetTheory.PGame.LF (xL i) y
                              theorem SetTheory.PGame.lf_of_mk_le {x : SetTheory.PGame} {yl : Type u_1} {yr : Type u_1} {yL : ylSetTheory.PGame} {yR : yrSetTheory.PGame} :
                              x SetTheory.PGame.mk yl yr yL yR∀ (j : yr), SetTheory.PGame.LF x (yR j)
                              theorem SetTheory.PGame.mk_lf_of_le {xl : Type u_1} {xr : Type u_1} {y : SetTheory.PGame} {j : xr} (xL : xlSetTheory.PGame) {xR : xrSetTheory.PGame} :
                              xR j ySetTheory.PGame.LF (SetTheory.PGame.mk xl xr xL xR) y
                              theorem SetTheory.PGame.lf_mk_of_le {x : SetTheory.PGame} {yl : Type u_1} {yr : Type u_1} {yL : ylSetTheory.PGame} (yR : yrSetTheory.PGame) {i : yl} :
                              x yL iSetTheory.PGame.LF x (SetTheory.PGame.mk yl yr yL yR)
                              Equations
                              • One or more equations did not get rendered due to their size.
                              instance SetTheory.PGame.instTransPGameLeLF :
                              Trans (fun (x x_1 : SetTheory.PGame) => x x_1) (fun (x x_1 : SetTheory.PGame) => SetTheory.PGame.LF x x_1) fun (x x_1 : SetTheory.PGame) => SetTheory.PGame.LF x x_1
                              Equations
                              instance SetTheory.PGame.instTransPGameLFLeLe :
                              Trans (fun (x x_1 : SetTheory.PGame) => SetTheory.PGame.LF x x_1) (fun (x x_1 : SetTheory.PGame) => x x_1) fun (x x_1 : SetTheory.PGame) => SetTheory.PGame.LF x x_1
                              Equations
                              theorem SetTheory.PGame.lf_mk {xl : Type u_1} {xr : Type u_1} (xL : xlSetTheory.PGame) (xR : xrSetTheory.PGame) (i : xl) :
                              theorem SetTheory.PGame.mk_lf {xl : Type u_1} {xr : Type u_1} (xL : xlSetTheory.PGame) (xR : xrSetTheory.PGame) (j : xr) :

                              This special case of PGame.le_of_forall_lf is useful when dealing with surreals, where < is preferred over .

                              The definition of 0 ≤ x on pre-games, in terms of 0 ⧏.

                              The definition of x ≤ 0 on pre-games, in terms of ⧏ 0.

                              The definition of 0 ⧏ x on pre-games, in terms of 0 ≤.

                              The definition of x ⧏ 0 on pre-games, in terms of ≤ 0.

                              The definition of 0 ≤ x on pre-games, in terms of 0 ≤ two moves later.

                              The definition of x ≤ 0 on pre-games, in terms of ≤ 0 two moves later.

                              The definition of 0 ⧏ x on pre-games, in terms of 0 ⧏ two moves later.

                              The definition of x ⧏ 0 on pre-games, in terms of ⧏ 0 two moves later.

                              Given a game won by the right player when they play second, provide a response to any move by left.

                              Equations
                              Instances For

                                Show that the response for right provided by rightResponse preserves the right-player-wins condition.

                                Given a game won by the left player when they play second, provide a response to any move by right.

                                Equations
                                Instances For

                                  Show that the response for left provided by leftResponse preserves the left-player-wins condition.

                                  A small family of pre-games is bounded above.

                                  A small set of pre-games is bounded above.

                                  A small family of pre-games is bounded below.

                                  A small set of pre-games is bounded below.

                                  The equivalence relation on pre-games. Two pre-games x, y are equivalent if x ≤ y and y ≤ x.

                                  If x ≈ 0, then the second player can always win x.

                                  Equations
                                  Instances For
                                    theorem SetTheory.PGame.le_of_le_of_equiv {x : SetTheory.PGame} {y : SetTheory.PGame} {z : SetTheory.PGame} (h₁ : x y) (h₂ : y z) :
                                    x z
                                    theorem SetTheory.PGame.le_congr_imp {x₁ : SetTheory.PGame} {y₁ : SetTheory.PGame} {x₂ : SetTheory.PGame} {y₂ : SetTheory.PGame} (hx : x₁ x₂) (hy : y₁ y₂) (h : x₁ y₁) :
                                    x₂ y₂
                                    theorem SetTheory.PGame.le_congr {x₁ : SetTheory.PGame} {y₁ : SetTheory.PGame} {x₂ : SetTheory.PGame} {y₂ : SetTheory.PGame} (hx : x₁ x₂) (hy : y₁ y₂) :
                                    x₁ y₁ x₂ y₂
                                    theorem SetTheory.PGame.le_congr_left {x₁ : SetTheory.PGame} {x₂ : SetTheory.PGame} {y : SetTheory.PGame} (hx : x₁ x₂) :
                                    x₁ y x₂ y
                                    theorem SetTheory.PGame.le_congr_right {x : SetTheory.PGame} {y₁ : SetTheory.PGame} {y₂ : SetTheory.PGame} (hy : y₁ y₂) :
                                    x y₁ x y₂
                                    theorem SetTheory.PGame.lf_congr {x₁ : SetTheory.PGame} {y₁ : SetTheory.PGame} {x₂ : SetTheory.PGame} {y₂ : SetTheory.PGame} (hx : x₁ x₂) (hy : y₁ y₂) :
                                    theorem SetTheory.PGame.lf_congr_imp {x₁ : SetTheory.PGame} {y₁ : SetTheory.PGame} {x₂ : SetTheory.PGame} {y₂ : SetTheory.PGame} (hx : x₁ x₂) (hy : y₁ y₂) :
                                    SetTheory.PGame.LF x₁ y₁SetTheory.PGame.LF x₂ y₂
                                    theorem SetTheory.PGame.lt_of_lt_of_equiv {x : SetTheory.PGame} {y : SetTheory.PGame} {z : SetTheory.PGame} (h₁ : x < y) (h₂ : y z) :
                                    x < z
                                    theorem SetTheory.PGame.lt_congr_imp {x₁ : SetTheory.PGame} {y₁ : SetTheory.PGame} {x₂ : SetTheory.PGame} {y₂ : SetTheory.PGame} (hx : x₁ x₂) (hy : y₁ y₂) (h : x₁ < y₁) :
                                    x₂ < y₂
                                    theorem SetTheory.PGame.lt_congr {x₁ : SetTheory.PGame} {y₁ : SetTheory.PGame} {x₂ : SetTheory.PGame} {y₂ : SetTheory.PGame} (hx : x₁ x₂) (hy : y₁ y₂) :
                                    x₁ < y₁ x₂ < y₂
                                    theorem SetTheory.PGame.lt_congr_left {x₁ : SetTheory.PGame} {x₂ : SetTheory.PGame} {y : SetTheory.PGame} (hx : x₁ x₂) :
                                    x₁ < y x₂ < y
                                    theorem SetTheory.PGame.lt_congr_right {x : SetTheory.PGame} {y₁ : SetTheory.PGame} {y₂ : SetTheory.PGame} (hy : y₁ y₂) :
                                    x < y₁ x < y₂
                                    theorem SetTheory.PGame.equiv_congr_left {y₁ : SetTheory.PGame} {y₂ : SetTheory.PGame} :
                                    y₁ y₂ ∀ (x₁ : SetTheory.PGame), x₁ y₁ x₁ y₂
                                    theorem SetTheory.PGame.equiv_congr_right {x₁ : SetTheory.PGame} {x₂ : SetTheory.PGame} :
                                    x₁ x₂ ∀ (y₁ : SetTheory.PGame), x₁ y₁ x₂ y₁

                                    The fuzzy, confused, or incomparable relation on pre-games.

                                    If x ‖ 0, then the first player can always win x.

                                    Equations
                                    Instances For

                                      The fuzzy, confused, or incomparable relation on pre-games.

                                      If x ‖ 0, then the first player can always win x.

                                      Equations
                                      • One or more equations did not get rendered due to their size.
                                      Instances For
                                        theorem SetTheory.PGame.fuzzy_congr {x₁ : SetTheory.PGame} {y₁ : SetTheory.PGame} {x₂ : SetTheory.PGame} {y₂ : SetTheory.PGame} (hx : x₁ x₂) (hy : y₁ y₂) :
                                        theorem SetTheory.PGame.fuzzy_congr_imp {x₁ : SetTheory.PGame} {y₁ : SetTheory.PGame} {x₂ : SetTheory.PGame} {y₂ : SetTheory.PGame} (hx : x₁ x₂) (hy : y₁ y₂) :

                                        Exactly one of the following is true (although we don't prove this here).

                                        Relabellings #

                                        Relabelling x y says that x and y are really the same game, just dressed up differently. Specifically, there is a bijection between the moves for Left in x and in y, and similarly for Right, and under these bijections we inductively have Relabellings for the consequent games.

                                        Instances For

                                          Relabelling x y says that x and y are really the same game, just dressed up differently. Specifically, there is a bijection between the moves for Left in x and in y, and similarly for Right, and under these bijections we inductively have Relabellings for the consequent games.

                                          Equations
                                          • One or more equations did not get rendered due to their size.
                                          Instances For

                                            The equivalence between left moves of x and y given by the relabelling.

                                            Equations
                                            Instances For

                                              The equivalence between right moves of x and y given by the relabelling.

                                              Equations
                                              Instances For

                                                A left move of x is a relabelling of a left move of y.

                                                Equations
                                                • One or more equations did not get rendered due to their size.
                                                Instances For

                                                  A right move of x is a relabelling of a right move of y.

                                                  Equations
                                                  • One or more equations did not get rendered due to their size.
                                                  Instances For

                                                    The identity relabelling.

                                                    Equations
                                                    • One or more equations did not get rendered due to their size.
                                                    Instances For

                                                      Flip a relabelling.

                                                      Equations
                                                      • One or more equations did not get rendered due to their size.
                                                      Instances For

                                                        A relabelling lets us prove equivalence of games.

                                                        Transitivity of relabelling.

                                                        Equations
                                                        • One or more equations did not get rendered due to their size.
                                                        Instances For

                                                          Any game without left or right moves is a relabelling of 0.

                                                          Equations
                                                          • One or more equations did not get rendered due to their size.
                                                          Instances For
                                                            Equations
                                                            • SetTheory.PGame.instCoeRelabellingEquivPGameInstHasEquivSetoid = { coe := }

                                                            Replace the types indexing the next moves for Left and Right by equivalent types.

                                                            Equations
                                                            Instances For

                                                              The game obtained by relabelling the next moves is a relabelling of the original game.

                                                              Equations
                                                              • One or more equations did not get rendered due to their size.
                                                              Instances For

                                                                Negation #

                                                                The negation of {L | R} is {-R | -L}.

                                                                Equations
                                                                Instances For
                                                                  @[simp]
                                                                  theorem SetTheory.PGame.neg_def {xl : Type u_1} {xr : Type u_1} {xL : xlSetTheory.PGame} {xR : xrSetTheory.PGame} :
                                                                  -SetTheory.PGame.mk xl xr xL xR = SetTheory.PGame.mk xr xl (fun (j : xr) => -xR j) fun (i : xl) => -xL i
                                                                  Equations
                                                                  • One or more equations did not get rendered due to their size.

                                                                  Turns a right move for x into a left move for -x and vice versa.

                                                                  Even though these types are the same (not definitionally so), this is the preferred way to convert between them.

                                                                  Equations
                                                                  Instances For

                                                                    Turns a left move for x into a right move for -x and vice versa.

                                                                    Even though these types are the same (not definitionally so), this is the preferred way to convert between them.

                                                                    Equations
                                                                    Instances For
                                                                      @[simp]
                                                                      @[simp]

                                                                      If x has the same moves as y, then -x has the same moves as -y.

                                                                      Equations
                                                                      • One or more equations did not get rendered due to their size.
                                                                      Instances For

                                                                        Addition and subtraction #

                                                                        The sum of x = {xL | xR} and y = {yL | yR} is {xL + y, x + yL | xR + y, x + yR}.

                                                                        Equations
                                                                        • One or more equations did not get rendered due to their size.

                                                                        The pre-game ((0+1)+⋯)+1.

                                                                        Equations
                                                                        @[simp]
                                                                        theorem SetTheory.PGame.nat_succ (n : ) :
                                                                        (n + 1) = n + 1

                                                                        x + 0 has exactly the same moves as x.

                                                                        Equations
                                                                        • One or more equations did not get rendered due to their size.
                                                                        Instances For

                                                                          x + 0 is equivalent to x.

                                                                          0 + x has exactly the same moves as x.

                                                                          Equations
                                                                          • One or more equations did not get rendered due to their size.
                                                                          Instances For

                                                                            0 + x is equivalent to x.

                                                                            Converts a left move for x or y into a left move for x + y and vice versa.

                                                                            Even though these types are the same (not definitionally so), this is the preferred way to convert between them.

                                                                            Equations
                                                                            Instances For

                                                                              Converts a right move for x or y into a right move for x + y and vice versa.

                                                                              Even though these types are the same (not definitionally so), this is the preferred way to convert between them.

                                                                              Equations
                                                                              Instances For
                                                                                @[simp]
                                                                                theorem SetTheory.PGame.mk_add_moveLeft_inl {xl : Type u_1} {xr : Type u_1} {yl : Type u_1} {yr : Type u_1} {xL : xlSetTheory.PGame} {xR : xrSetTheory.PGame} {yL : ylSetTheory.PGame} {yR : yrSetTheory.PGame} {i : xl} :
                                                                                @[simp]
                                                                                theorem SetTheory.PGame.mk_add_moveRight_inl {xl : Type u_1} {xr : Type u_1} {yl : Type u_1} {yr : Type u_1} {xL : xlSetTheory.PGame} {xR : xrSetTheory.PGame} {yL : ylSetTheory.PGame} {yR : yrSetTheory.PGame} {i : xr} :
                                                                                @[simp]
                                                                                theorem SetTheory.PGame.mk_add_moveLeft_inr {xl : Type u_1} {xr : Type u_1} {yl : Type u_1} {yr : Type u_1} {xL : xlSetTheory.PGame} {xR : xrSetTheory.PGame} {yL : ylSetTheory.PGame} {yR : yrSetTheory.PGame} {i : yl} :
                                                                                @[simp]
                                                                                theorem SetTheory.PGame.mk_add_moveRight_inr {xl : Type u_1} {xr : Type u_1} {yl : Type u_1} {yr : Type u_1} {xL : xlSetTheory.PGame} {xR : xrSetTheory.PGame} {yL : ylSetTheory.PGame} {yR : yrSetTheory.PGame} {i : yr} :
                                                                                theorem SetTheory.PGame.leftMoves_add_cases {x : SetTheory.PGame} {y : SetTheory.PGame} (k : SetTheory.PGame.LeftMoves (x + y)) {P : SetTheory.PGame.LeftMoves (x + y)Prop} (hl : ∀ (i : SetTheory.PGame.LeftMoves x), P (SetTheory.PGame.toLeftMovesAdd (Sum.inl i))) (hr : ∀ (i : SetTheory.PGame.LeftMoves y), P (SetTheory.PGame.toLeftMovesAdd (Sum.inr i))) :
                                                                                P k
                                                                                theorem SetTheory.PGame.rightMoves_add_cases {x : SetTheory.PGame} {y : SetTheory.PGame} (k : SetTheory.PGame.RightMoves (x + y)) {P : SetTheory.PGame.RightMoves (x + y)Prop} (hl : ∀ (j : SetTheory.PGame.RightMoves x), P (SetTheory.PGame.toRightMovesAdd (Sum.inl j))) (hr : ∀ (j : SetTheory.PGame.RightMoves y), P (SetTheory.PGame.toRightMovesAdd (Sum.inr j))) :
                                                                                P k

                                                                                If w has the same moves as x and y has the same moves as z, then w + y has the same moves as x + z.

                                                                                Equations
                                                                                • One or more equations did not get rendered due to their size.
                                                                                Instances For
                                                                                  @[simp]

                                                                                  If w has the same moves as x and y has the same moves as z, then w - y has the same moves as x - z.

                                                                                  Equations
                                                                                  Instances For

                                                                                    -(x + y) has exactly the same moves as -x + -y.

                                                                                    Equations
                                                                                    • One or more equations did not get rendered due to their size.
                                                                                    Instances For

                                                                                      x + y has exactly the same moves as y + x.

                                                                                      Equations
                                                                                      • One or more equations did not get rendered due to their size.
                                                                                      Instances For

                                                                                        (x + y) + z has exactly the same moves as x + (y + z).

                                                                                        Equations
                                                                                        • One or more equations did not get rendered due to their size.
                                                                                        Instances For
                                                                                          theorem SetTheory.PGame.add_congr {w : SetTheory.PGame} {x : SetTheory.PGame} {y : SetTheory.PGame} {z : SetTheory.PGame} (h₁ : w x) (h₂ : y z) :
                                                                                          w + y x + z
                                                                                          theorem SetTheory.PGame.sub_congr {w : SetTheory.PGame} {x : SetTheory.PGame} {y : SetTheory.PGame} {z : SetTheory.PGame} (h₁ : w x) (h₂ : y z) :
                                                                                          w - y x - z

                                                                                          Special pre-games #

                                                                                          The pre-game star, which is fuzzy with zero.

                                                                                          Equations
                                                                                          Instances For