state
stringlengths
0
159k
srcUpToTactic
stringlengths
387
167k
nextTactic
stringlengths
3
9k
declUpToTactic
stringlengths
22
11.5k
declId
stringlengths
38
95
decl
stringlengths
16
1.89k
file_tag
stringlengths
17
73
x✝ : PGame inst✝ : Impartial x✝ G : PGame := x✝ i : LeftMoves (x✝ + nim (grundyValue x✝)) i₂ : LeftMoves (mk (Quotient.out (grundyValue x✝)).α (Quotient.out (grundyValue x✝)).α (fun o₂ => nim (typein (fun x x_1 => x < x_1) o₂)) fun o₂ => nim (typein (fun x x_1 => x < x_1) o₂)) ⊢ ∃ i, grundyValue (moveLeft G i) = typein (Quotient.out (grundyValue G)).r i₂
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by
revert i₂
/-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by
Mathlib.SetTheory.Game.Nim.271_0.mmFMhRYSjViKjcP
/-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h
Mathlib_SetTheory_Game_Nim
x✝ : PGame inst✝ : Impartial x✝ G : PGame := x✝ i : LeftMoves (x✝ + nim (grundyValue x✝)) ⊢ ∀ (i₂ : LeftMoves (mk (Quotient.out (grundyValue x✝)).α (Quotient.out (grundyValue x✝)).α (fun o₂ => nim (typein (fun x x_1 => x < x_1) o₂)) fun o₂ => nim (typein (fun x x_1 => x < x_1) o₂))), ∃ i, grundyValue (moveLeft G i) = typein (Quotient.out (grundyValue G)).r i₂
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂
rw [grundyValue_eq_mex_left]
/-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂
Mathlib.SetTheory.Game.Nim.271_0.mmFMhRYSjViKjcP
/-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h
Mathlib_SetTheory_Game_Nim
x✝ : PGame inst✝ : Impartial x✝ G : PGame := x✝ i : LeftMoves (x✝ + nim (grundyValue x✝)) ⊢ ∀ (i₂ : LeftMoves (mk (Quotient.out (mex fun i => grundyValue (moveLeft x✝ i))).α (Quotient.out (mex fun i => grundyValue (moveLeft x✝ i))).α (fun o₂ => nim (typein (fun x x_1 => x < x_1) o₂)) fun o₂ => nim (typein (fun x x_1 => x < x_1) o₂))), ∃ i, grundyValue (moveLeft G i) = typein (Quotient.out (mex fun i => grundyValue (moveLeft x✝ i))).r i₂
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left]
intro i₂
/-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left]
Mathlib.SetTheory.Game.Nim.271_0.mmFMhRYSjViKjcP
/-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h
Mathlib_SetTheory_Game_Nim
x✝ : PGame inst✝ : Impartial x✝ G : PGame := x✝ i : LeftMoves (x✝ + nim (grundyValue x✝)) i₂ : LeftMoves (mk (Quotient.out (mex fun i => grundyValue (moveLeft x✝ i))).α (Quotient.out (mex fun i => grundyValue (moveLeft x✝ i))).α (fun o₂ => nim (typein (fun x x_1 => x < x_1) o₂)) fun o₂ => nim (typein (fun x x_1 => x < x_1) o₂)) ⊢ ∃ i, grundyValue (moveLeft G i) = typein (Quotient.out (mex fun i => grundyValue (moveLeft x✝ i))).r i₂
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂
have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin)
/-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂
Mathlib.SetTheory.Game.Nim.271_0.mmFMhRYSjViKjcP
/-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h
Mathlib_SetTheory_Game_Nim
x✝ : PGame inst✝ : Impartial x✝ G : PGame := x✝ i : LeftMoves (x✝ + nim (grundyValue x✝)) i₂ : LeftMoves (mk (Quotient.out (mex fun i => grundyValue (moveLeft x✝ i))).α (Quotient.out (mex fun i => grundyValue (moveLeft x✝ i))).α (fun o₂ => nim (typein (fun x x_1 => x < x_1) o₂)) fun o₂ => nim (typein (fun x x_1 => x < x_1) o₂)) hnotin : typein (fun x x_1 => x < x_1) i₂ ∉ (Set.range fun i => grundyValue (moveLeft x✝ i))ᶜ ⊢ ∃ i, grundyValue (moveLeft G i) = typein (Quotient.out (mex fun i => grundyValue (moveLeft x✝ i))).r i₂
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin)
simpa using hnotin
/-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin)
Mathlib.SetTheory.Game.Nim.271_0.mmFMhRYSjViKjcP
/-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h
Mathlib_SetTheory_Game_Nim
case hr x✝ : PGame inst✝ : Impartial x✝ G : PGame := x✝ i : LeftMoves (x✝ + nim (grundyValue x✝)) i₂ : LeftMoves (mk (Quotient.out (grundyValue x✝)).α (Quotient.out (grundyValue x✝)).α (fun o₂ => nim (typein (fun x x_1 => x < x_1) o₂)) fun o₂ => nim (typein (fun x x_1 => x < x_1) o₂)) h' : ∃ i, grundyValue (moveLeft G i) = typein (Quotient.out (grundyValue G)).r i₂ ⊢ ∃ i, moveLeft (x✝ + moveLeft (mk (Quotient.out (grundyValue x✝)).α (Quotient.out (grundyValue x✝)).α (fun o₂ => nim (typein (fun x x_1 => x < x_1) o₂)) fun o₂ => nim (typein (fun x x_1 => x < x_1) o₂)) i₂) i ≈ 0
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin
cases' h' with i hi
/-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin
Mathlib.SetTheory.Game.Nim.271_0.mmFMhRYSjViKjcP
/-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h
Mathlib_SetTheory_Game_Nim
case hr.intro x✝ : PGame inst✝ : Impartial x✝ G : PGame := x✝ i✝ : LeftMoves (x✝ + nim (grundyValue x✝)) i₂ : LeftMoves (mk (Quotient.out (grundyValue x✝)).α (Quotient.out (grundyValue x✝)).α (fun o₂ => nim (typein (fun x x_1 => x < x_1) o₂)) fun o₂ => nim (typein (fun x x_1 => x < x_1) o₂)) i : LeftMoves G hi : grundyValue (moveLeft G i) = typein (Quotient.out (grundyValue G)).r i₂ ⊢ ∃ i, moveLeft (x✝ + moveLeft (mk (Quotient.out (grundyValue x✝)).α (Quotient.out (grundyValue x✝)).α (fun o₂ => nim (typein (fun x x_1 => x < x_1) o₂)) fun o₂ => nim (typein (fun x x_1 => x < x_1) o₂)) i₂) i ≈ 0
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi
use toLeftMovesAdd (Sum.inl i)
/-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi
Mathlib.SetTheory.Game.Nim.271_0.mmFMhRYSjViKjcP
/-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h
Mathlib_SetTheory_Game_Nim
case h x✝ : PGame inst✝ : Impartial x✝ G : PGame := x✝ i✝ : LeftMoves (x✝ + nim (grundyValue x✝)) i₂ : LeftMoves (mk (Quotient.out (grundyValue x✝)).α (Quotient.out (grundyValue x✝)).α (fun o₂ => nim (typein (fun x x_1 => x < x_1) o₂)) fun o₂ => nim (typein (fun x x_1 => x < x_1) o₂)) i : LeftMoves G hi : grundyValue (moveLeft G i) = typein (Quotient.out (grundyValue G)).r i₂ ⊢ moveLeft (x✝ + moveLeft (mk (Quotient.out (grundyValue x✝)).α (Quotient.out (grundyValue x✝)).α (fun o₂ => nim (typein (fun x x_1 => x < x_1) o₂)) fun o₂ => nim (typein (fun x x_1 => x < x_1) o₂)) i₂) (toLeftMovesAdd (Sum.inl i)) ≈ 0
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i)
rw [add_moveLeft_inl, moveLeft_mk]
/-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i)
Mathlib.SetTheory.Game.Nim.271_0.mmFMhRYSjViKjcP
/-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h
Mathlib_SetTheory_Game_Nim
case h x✝ : PGame inst✝ : Impartial x✝ G : PGame := x✝ i✝ : LeftMoves (x✝ + nim (grundyValue x✝)) i₂ : LeftMoves (mk (Quotient.out (grundyValue x✝)).α (Quotient.out (grundyValue x✝)).α (fun o₂ => nim (typein (fun x x_1 => x < x_1) o₂)) fun o₂ => nim (typein (fun x x_1 => x < x_1) o₂)) i : LeftMoves G hi : grundyValue (moveLeft G i) = typein (Quotient.out (grundyValue G)).r i₂ ⊢ moveLeft x✝ i + nim (typein (fun x x_1 => x < x_1) i₂) ≈ 0
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk]
apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i)))
/-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk]
Mathlib.SetTheory.Game.Nim.271_0.mmFMhRYSjViKjcP
/-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h
Mathlib_SetTheory_Game_Nim
case h x✝ : PGame inst✝ : Impartial x✝ G : PGame := x✝ i✝ : LeftMoves (x✝ + nim (grundyValue x✝)) i₂ : LeftMoves (mk (Quotient.out (grundyValue x✝)).α (Quotient.out (grundyValue x✝)).α (fun o₂ => nim (typein (fun x x_1 => x < x_1) o₂)) fun o₂ => nim (typein (fun x x_1 => x < x_1) o₂)) i : LeftMoves G hi : grundyValue (moveLeft G i) = typein (Quotient.out (grundyValue G)).r i₂ ⊢ nim (grundyValue (moveLeft G i)) + nim (typein (fun x x_1 => x < x_1) i₂) ≈ 0
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i)))
simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i)))
/-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i)))
Mathlib.SetTheory.Game.Nim.271_0.mmFMhRYSjViKjcP
/-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h
Mathlib_SetTheory_Game_Nim
x✝ : PGame inst✝ : Impartial x✝ a✝ : ∀ (y : (x : PGame) ×' Impartial x), (invImage (fun a => PSigma.casesOn a fun G snd => G) instWellFoundedRelationPGame).1 y { fst := x✝, snd := inst✝ } → y.1 ≈ nim (grundyValue y.1) G : PGame := x✝ i₁ : LeftMoves x✝ ⊢ (invImage (fun a => PSigma.casesOn a fun G snd => G) instWellFoundedRelationPGame).1 { fst := moveLeft G i₁, snd := (_ : Impartial (moveLeft G i₁)) } { fst := x✝, snd := inst✝ }
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by
pgame_wf_tac
/-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by
Mathlib.SetTheory.Game.Nim.271_0.mmFMhRYSjViKjcP
/-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h
Mathlib_SetTheory_Game_Nim
x✝ : PGame inst✝ : Impartial x✝ a✝ : ∀ (y : (x : PGame) ×' Impartial x), (invImage (fun a => PSigma.casesOn a fun G snd => G) instWellFoundedRelationPGame).1 y { fst := x✝, snd := inst✝ } → y.1 ≈ nim (grundyValue y.1) G : PGame := x✝ i₂ : LeftMoves (mk (Quotient.out (grundyValue x✝)).α (Quotient.out (grundyValue x✝)).α (fun o₂ => nim (typein (fun x x_1 => x < x_1) o₂)) fun o₂ => nim (typein (fun x x_1 => x < x_1) o₂)) h' : ∃ i, grundyValue (moveLeft G i) = typein (Quotient.out (grundyValue G)).r i₂ i : LeftMoves G hi : grundyValue (moveLeft G i) = typein (Quotient.out (grundyValue G)).r i₂ h✝ : h' = (_ : ∃ i, grundyValue (moveLeft G i) = typein (Quotient.out (grundyValue G)).r i₂) ⊢ (invImage (fun a => PSigma.casesOn a fun G snd => G) instWellFoundedRelationPGame).1 { fst := moveLeft G i, snd := (_ : Impartial (moveLeft G i)) } { fst := x✝, snd := inst✝ }
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by
pgame_wf_tac
/-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by
Mathlib.SetTheory.Game.Nim.271_0.mmFMhRYSjViKjcP
/-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h
Mathlib_SetTheory_Game_Nim
G : PGame inst✝ : Impartial G o : Ordinal.{u_1} ⊢ grundyValue G = o → G ≈ nim o
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by
rintro rfl
theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by
Mathlib.SetTheory.Game.Nim.312_0.mmFMhRYSjViKjcP
theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o)
Mathlib_SetTheory_Game_Nim
G : PGame inst✝ : Impartial G ⊢ G ≈ nim (grundyValue G)
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl;
exact equiv_nim_grundyValue G
theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl;
Mathlib.SetTheory.Game.Nim.312_0.mmFMhRYSjViKjcP
theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o)
Mathlib_SetTheory_Game_Nim
G : PGame inst✝ : Impartial G o : Ordinal.{u_1} ⊢ G ≈ nim o → grundyValue G = o
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by
intro h
theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by
Mathlib.SetTheory.Game.Nim.312_0.mmFMhRYSjViKjcP
theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o)
Mathlib_SetTheory_Game_Nim
G : PGame inst✝ : Impartial G o : Ordinal.{u_1} h : G ≈ nim o ⊢ grundyValue G = o
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h;
rw [← nim_equiv_iff_eq]
theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h;
Mathlib.SetTheory.Game.Nim.312_0.mmFMhRYSjViKjcP
theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o)
Mathlib_SetTheory_Game_Nim
G : PGame inst✝ : Impartial G o : Ordinal.{u_1} h : G ≈ nim o ⊢ nim (grundyValue G) ≈ nim o
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq];
exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h
theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq];
Mathlib.SetTheory.Game.Nim.312_0.mmFMhRYSjViKjcP
theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o)
Mathlib_SetTheory_Game_Nim
G : PGame inst✝ : Impartial G ⊢ grundyValue G = 0 ↔ G ≈ 0
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq]; exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h⟩ #align pgame.grundy_value_eq_iff_equiv_nim SetTheory.PGame.grundyValue_eq_iff_equiv_nim @[simp] theorem nim_grundyValue (o : Ordinal.{u}) : grundyValue (nim o) = o := grundyValue_eq_iff_equiv_nim.2 PGame.equiv_rfl #align pgame.nim_grundy_value SetTheory.PGame.nim_grundyValue theorem grundyValue_eq_iff_equiv (G H : PGame) [G.Impartial] [H.Impartial] : grundyValue G = grundyValue H ↔ (G ≈ H) := grundyValue_eq_iff_equiv_nim.trans (equiv_congr_left.1 (equiv_nim_grundyValue H) _).symm #align pgame.grundy_value_eq_iff_equiv SetTheory.PGame.grundyValue_eq_iff_equiv @[simp] theorem grundyValue_zero : grundyValue 0 = 0 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_zero_equiv) #align pgame.grundy_value_zero SetTheory.PGame.grundyValue_zero theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by
rw [← grundyValue_eq_iff_equiv, grundyValue_zero]
theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by
Mathlib.SetTheory.Game.Nim.333_0.mmFMhRYSjViKjcP
theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0)
Mathlib_SetTheory_Game_Nim
G : PGame inst✝ : Impartial G ⊢ grundyValue (-G) = grundyValue G
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq]; exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h⟩ #align pgame.grundy_value_eq_iff_equiv_nim SetTheory.PGame.grundyValue_eq_iff_equiv_nim @[simp] theorem nim_grundyValue (o : Ordinal.{u}) : grundyValue (nim o) = o := grundyValue_eq_iff_equiv_nim.2 PGame.equiv_rfl #align pgame.nim_grundy_value SetTheory.PGame.nim_grundyValue theorem grundyValue_eq_iff_equiv (G H : PGame) [G.Impartial] [H.Impartial] : grundyValue G = grundyValue H ↔ (G ≈ H) := grundyValue_eq_iff_equiv_nim.trans (equiv_congr_left.1 (equiv_nim_grundyValue H) _).symm #align pgame.grundy_value_eq_iff_equiv SetTheory.PGame.grundyValue_eq_iff_equiv @[simp] theorem grundyValue_zero : grundyValue 0 = 0 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_zero_equiv) #align pgame.grundy_value_zero SetTheory.PGame.grundyValue_zero theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by rw [← grundyValue_eq_iff_equiv, grundyValue_zero] #align pgame.grundy_value_iff_equiv_zero SetTheory.PGame.grundyValue_iff_equiv_zero @[simp] theorem grundyValue_star : grundyValue star = 1 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_one_equiv) #align pgame.grundy_value_star SetTheory.PGame.grundyValue_star @[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G := by
rw [grundyValue_eq_iff_equiv_nim, neg_equiv_iff, neg_nim, ← grundyValue_eq_iff_equiv_nim]
@[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G := by
Mathlib.SetTheory.Game.Nim.342_0.mmFMhRYSjViKjcP
@[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G
Mathlib_SetTheory_Game_Nim
l r : Type u L : l → PGame R : r → PGame x✝ : Impartial (mk l r L R) ⊢ grundyValue (mk l r L R) = mex fun i => grundyValue (moveRight (mk l r L R) i)
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq]; exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h⟩ #align pgame.grundy_value_eq_iff_equiv_nim SetTheory.PGame.grundyValue_eq_iff_equiv_nim @[simp] theorem nim_grundyValue (o : Ordinal.{u}) : grundyValue (nim o) = o := grundyValue_eq_iff_equiv_nim.2 PGame.equiv_rfl #align pgame.nim_grundy_value SetTheory.PGame.nim_grundyValue theorem grundyValue_eq_iff_equiv (G H : PGame) [G.Impartial] [H.Impartial] : grundyValue G = grundyValue H ↔ (G ≈ H) := grundyValue_eq_iff_equiv_nim.trans (equiv_congr_left.1 (equiv_nim_grundyValue H) _).symm #align pgame.grundy_value_eq_iff_equiv SetTheory.PGame.grundyValue_eq_iff_equiv @[simp] theorem grundyValue_zero : grundyValue 0 = 0 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_zero_equiv) #align pgame.grundy_value_zero SetTheory.PGame.grundyValue_zero theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by rw [← grundyValue_eq_iff_equiv, grundyValue_zero] #align pgame.grundy_value_iff_equiv_zero SetTheory.PGame.grundyValue_iff_equiv_zero @[simp] theorem grundyValue_star : grundyValue star = 1 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_one_equiv) #align pgame.grundy_value_star SetTheory.PGame.grundyValue_star @[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G := by rw [grundyValue_eq_iff_equiv_nim, neg_equiv_iff, neg_nim, ← grundyValue_eq_iff_equiv_nim] #align pgame.grundy_value_neg SetTheory.PGame.grundyValue_neg theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by
rw [← grundyValue_neg, grundyValue_eq_mex_left]
theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by
Mathlib.SetTheory.Game.Nim.347_0.mmFMhRYSjViKjcP
theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i haveI : (R i).Impartial
Mathlib_SetTheory_Game_Nim
l r : Type u L : l → PGame R : r → PGame x✝ : Impartial (mk l r L R) ⊢ (mex fun i => grundyValue (moveLeft (-mk l r L R) i)) = mex fun i => grundyValue (moveRight (mk l r L R) i)
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq]; exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h⟩ #align pgame.grundy_value_eq_iff_equiv_nim SetTheory.PGame.grundyValue_eq_iff_equiv_nim @[simp] theorem nim_grundyValue (o : Ordinal.{u}) : grundyValue (nim o) = o := grundyValue_eq_iff_equiv_nim.2 PGame.equiv_rfl #align pgame.nim_grundy_value SetTheory.PGame.nim_grundyValue theorem grundyValue_eq_iff_equiv (G H : PGame) [G.Impartial] [H.Impartial] : grundyValue G = grundyValue H ↔ (G ≈ H) := grundyValue_eq_iff_equiv_nim.trans (equiv_congr_left.1 (equiv_nim_grundyValue H) _).symm #align pgame.grundy_value_eq_iff_equiv SetTheory.PGame.grundyValue_eq_iff_equiv @[simp] theorem grundyValue_zero : grundyValue 0 = 0 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_zero_equiv) #align pgame.grundy_value_zero SetTheory.PGame.grundyValue_zero theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by rw [← grundyValue_eq_iff_equiv, grundyValue_zero] #align pgame.grundy_value_iff_equiv_zero SetTheory.PGame.grundyValue_iff_equiv_zero @[simp] theorem grundyValue_star : grundyValue star = 1 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_one_equiv) #align pgame.grundy_value_star SetTheory.PGame.grundyValue_star @[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G := by rw [grundyValue_eq_iff_equiv_nim, neg_equiv_iff, neg_nim, ← grundyValue_eq_iff_equiv_nim] #align pgame.grundy_value_neg SetTheory.PGame.grundyValue_neg theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left]
congr
theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left]
Mathlib.SetTheory.Game.Nim.347_0.mmFMhRYSjViKjcP
theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i haveI : (R i).Impartial
Mathlib_SetTheory_Game_Nim
case e_f l r : Type u L : l → PGame R : r → PGame x✝ : Impartial (mk l r L R) ⊢ (fun i => grundyValue (moveLeft (-mk l r L R) i)) = fun i => grundyValue (moveRight (mk l r L R) i)
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq]; exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h⟩ #align pgame.grundy_value_eq_iff_equiv_nim SetTheory.PGame.grundyValue_eq_iff_equiv_nim @[simp] theorem nim_grundyValue (o : Ordinal.{u}) : grundyValue (nim o) = o := grundyValue_eq_iff_equiv_nim.2 PGame.equiv_rfl #align pgame.nim_grundy_value SetTheory.PGame.nim_grundyValue theorem grundyValue_eq_iff_equiv (G H : PGame) [G.Impartial] [H.Impartial] : grundyValue G = grundyValue H ↔ (G ≈ H) := grundyValue_eq_iff_equiv_nim.trans (equiv_congr_left.1 (equiv_nim_grundyValue H) _).symm #align pgame.grundy_value_eq_iff_equiv SetTheory.PGame.grundyValue_eq_iff_equiv @[simp] theorem grundyValue_zero : grundyValue 0 = 0 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_zero_equiv) #align pgame.grundy_value_zero SetTheory.PGame.grundyValue_zero theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by rw [← grundyValue_eq_iff_equiv, grundyValue_zero] #align pgame.grundy_value_iff_equiv_zero SetTheory.PGame.grundyValue_iff_equiv_zero @[simp] theorem grundyValue_star : grundyValue star = 1 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_one_equiv) #align pgame.grundy_value_star SetTheory.PGame.grundyValue_star @[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G := by rw [grundyValue_eq_iff_equiv_nim, neg_equiv_iff, neg_nim, ← grundyValue_eq_iff_equiv_nim] #align pgame.grundy_value_neg SetTheory.PGame.grundyValue_neg theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr
ext i
theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr
Mathlib.SetTheory.Game.Nim.347_0.mmFMhRYSjViKjcP
theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i haveI : (R i).Impartial
Mathlib_SetTheory_Game_Nim
case e_f.h l r : Type u L : l → PGame R : r → PGame x✝ : Impartial (mk l r L R) i : LeftMoves (-mk l r L R) ⊢ grundyValue (moveLeft (-mk l r L R) i) = grundyValue (moveRight (mk l r L R) i)
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq]; exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h⟩ #align pgame.grundy_value_eq_iff_equiv_nim SetTheory.PGame.grundyValue_eq_iff_equiv_nim @[simp] theorem nim_grundyValue (o : Ordinal.{u}) : grundyValue (nim o) = o := grundyValue_eq_iff_equiv_nim.2 PGame.equiv_rfl #align pgame.nim_grundy_value SetTheory.PGame.nim_grundyValue theorem grundyValue_eq_iff_equiv (G H : PGame) [G.Impartial] [H.Impartial] : grundyValue G = grundyValue H ↔ (G ≈ H) := grundyValue_eq_iff_equiv_nim.trans (equiv_congr_left.1 (equiv_nim_grundyValue H) _).symm #align pgame.grundy_value_eq_iff_equiv SetTheory.PGame.grundyValue_eq_iff_equiv @[simp] theorem grundyValue_zero : grundyValue 0 = 0 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_zero_equiv) #align pgame.grundy_value_zero SetTheory.PGame.grundyValue_zero theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by rw [← grundyValue_eq_iff_equiv, grundyValue_zero] #align pgame.grundy_value_iff_equiv_zero SetTheory.PGame.grundyValue_iff_equiv_zero @[simp] theorem grundyValue_star : grundyValue star = 1 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_one_equiv) #align pgame.grundy_value_star SetTheory.PGame.grundyValue_star @[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G := by rw [grundyValue_eq_iff_equiv_nim, neg_equiv_iff, neg_nim, ← grundyValue_eq_iff_equiv_nim] #align pgame.grundy_value_neg SetTheory.PGame.grundyValue_neg theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i
haveI : (R i).Impartial := @Impartial.moveRight_impartial ⟨l, r, L, R⟩ _ i
theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i
Mathlib.SetTheory.Game.Nim.347_0.mmFMhRYSjViKjcP
theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i haveI : (R i).Impartial
Mathlib_SetTheory_Game_Nim
case e_f.h l r : Type u L : l → PGame R : r → PGame x✝ : Impartial (mk l r L R) i : LeftMoves (-mk l r L R) this : Impartial (R i) ⊢ grundyValue (moveLeft (-mk l r L R) i) = grundyValue (moveRight (mk l r L R) i)
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq]; exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h⟩ #align pgame.grundy_value_eq_iff_equiv_nim SetTheory.PGame.grundyValue_eq_iff_equiv_nim @[simp] theorem nim_grundyValue (o : Ordinal.{u}) : grundyValue (nim o) = o := grundyValue_eq_iff_equiv_nim.2 PGame.equiv_rfl #align pgame.nim_grundy_value SetTheory.PGame.nim_grundyValue theorem grundyValue_eq_iff_equiv (G H : PGame) [G.Impartial] [H.Impartial] : grundyValue G = grundyValue H ↔ (G ≈ H) := grundyValue_eq_iff_equiv_nim.trans (equiv_congr_left.1 (equiv_nim_grundyValue H) _).symm #align pgame.grundy_value_eq_iff_equiv SetTheory.PGame.grundyValue_eq_iff_equiv @[simp] theorem grundyValue_zero : grundyValue 0 = 0 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_zero_equiv) #align pgame.grundy_value_zero SetTheory.PGame.grundyValue_zero theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by rw [← grundyValue_eq_iff_equiv, grundyValue_zero] #align pgame.grundy_value_iff_equiv_zero SetTheory.PGame.grundyValue_iff_equiv_zero @[simp] theorem grundyValue_star : grundyValue star = 1 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_one_equiv) #align pgame.grundy_value_star SetTheory.PGame.grundyValue_star @[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G := by rw [grundyValue_eq_iff_equiv_nim, neg_equiv_iff, neg_nim, ← grundyValue_eq_iff_equiv_nim] #align pgame.grundy_value_neg SetTheory.PGame.grundyValue_neg theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i haveI : (R i).Impartial := @Impartial.moveRight_impartial ⟨l, r, L, R⟩ _ i
apply grundyValue_neg
theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i haveI : (R i).Impartial := @Impartial.moveRight_impartial ⟨l, r, L, R⟩ _ i
Mathlib.SetTheory.Game.Nim.347_0.mmFMhRYSjViKjcP
theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i haveI : (R i).Impartial
Mathlib_SetTheory_Game_Nim
n m : ℕ ⊢ grundyValue (nim ↑n + nim ↑m) = ↑(n ^^^ m)
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq]; exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h⟩ #align pgame.grundy_value_eq_iff_equiv_nim SetTheory.PGame.grundyValue_eq_iff_equiv_nim @[simp] theorem nim_grundyValue (o : Ordinal.{u}) : grundyValue (nim o) = o := grundyValue_eq_iff_equiv_nim.2 PGame.equiv_rfl #align pgame.nim_grundy_value SetTheory.PGame.nim_grundyValue theorem grundyValue_eq_iff_equiv (G H : PGame) [G.Impartial] [H.Impartial] : grundyValue G = grundyValue H ↔ (G ≈ H) := grundyValue_eq_iff_equiv_nim.trans (equiv_congr_left.1 (equiv_nim_grundyValue H) _).symm #align pgame.grundy_value_eq_iff_equiv SetTheory.PGame.grundyValue_eq_iff_equiv @[simp] theorem grundyValue_zero : grundyValue 0 = 0 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_zero_equiv) #align pgame.grundy_value_zero SetTheory.PGame.grundyValue_zero theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by rw [← grundyValue_eq_iff_equiv, grundyValue_zero] #align pgame.grundy_value_iff_equiv_zero SetTheory.PGame.grundyValue_iff_equiv_zero @[simp] theorem grundyValue_star : grundyValue star = 1 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_one_equiv) #align pgame.grundy_value_star SetTheory.PGame.grundyValue_star @[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G := by rw [grundyValue_eq_iff_equiv_nim, neg_equiv_iff, neg_nim, ← grundyValue_eq_iff_equiv_nim] #align pgame.grundy_value_neg SetTheory.PGame.grundyValue_neg theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i haveI : (R i).Impartial := @Impartial.moveRight_impartial ⟨l, r, L, R⟩ _ i apply grundyValue_neg #align pgame.grundy_value_eq_mex_right SetTheory.PGame.grundyValue_eq_mex_right -- Todo: this actually generalizes to all ordinals, by defining `Ordinal.lxor` as the pairwise -- `Nat.xor` of base `ω` Cantor normal forms. /-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables.
induction' n using Nat.strong_induction_on with n hn generalizing m
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables.
Mathlib.SetTheory.Game.Nim.360_0.mmFMhRYSjViKjcP
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m
Mathlib_SetTheory_Game_Nim
case h n : ℕ hn : ∀ m < n, ∀ (m_1 : ℕ), grundyValue (nim ↑m + nim ↑m_1) = ↑(m ^^^ m_1) m : ℕ ⊢ grundyValue (nim ↑n + nim ↑m) = ↑(n ^^^ m)
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq]; exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h⟩ #align pgame.grundy_value_eq_iff_equiv_nim SetTheory.PGame.grundyValue_eq_iff_equiv_nim @[simp] theorem nim_grundyValue (o : Ordinal.{u}) : grundyValue (nim o) = o := grundyValue_eq_iff_equiv_nim.2 PGame.equiv_rfl #align pgame.nim_grundy_value SetTheory.PGame.nim_grundyValue theorem grundyValue_eq_iff_equiv (G H : PGame) [G.Impartial] [H.Impartial] : grundyValue G = grundyValue H ↔ (G ≈ H) := grundyValue_eq_iff_equiv_nim.trans (equiv_congr_left.1 (equiv_nim_grundyValue H) _).symm #align pgame.grundy_value_eq_iff_equiv SetTheory.PGame.grundyValue_eq_iff_equiv @[simp] theorem grundyValue_zero : grundyValue 0 = 0 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_zero_equiv) #align pgame.grundy_value_zero SetTheory.PGame.grundyValue_zero theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by rw [← grundyValue_eq_iff_equiv, grundyValue_zero] #align pgame.grundy_value_iff_equiv_zero SetTheory.PGame.grundyValue_iff_equiv_zero @[simp] theorem grundyValue_star : grundyValue star = 1 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_one_equiv) #align pgame.grundy_value_star SetTheory.PGame.grundyValue_star @[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G := by rw [grundyValue_eq_iff_equiv_nim, neg_equiv_iff, neg_nim, ← grundyValue_eq_iff_equiv_nim] #align pgame.grundy_value_neg SetTheory.PGame.grundyValue_neg theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i haveI : (R i).Impartial := @Impartial.moveRight_impartial ⟨l, r, L, R⟩ _ i apply grundyValue_neg #align pgame.grundy_value_eq_mex_right SetTheory.PGame.grundyValue_eq_mex_right -- Todo: this actually generalizes to all ordinals, by defining `Ordinal.lxor` as the pairwise -- `Nat.xor` of base `ω` Cantor normal forms. /-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m
induction' m using Nat.strong_induction_on with m hm
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m
Mathlib.SetTheory.Game.Nim.360_0.mmFMhRYSjViKjcP
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m
Mathlib_SetTheory_Game_Nim
case h.h n : ℕ hn : ∀ m < n, ∀ (m_1 : ℕ), grundyValue (nim ↑m + nim ↑m_1) = ↑(m ^^^ m_1) m : ℕ hm : ∀ m_1 < m, grundyValue (nim ↑n + nim ↑m_1) = ↑(n ^^^ m_1) ⊢ grundyValue (nim ↑n + nim ↑m) = ↑(n ^^^ m)
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq]; exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h⟩ #align pgame.grundy_value_eq_iff_equiv_nim SetTheory.PGame.grundyValue_eq_iff_equiv_nim @[simp] theorem nim_grundyValue (o : Ordinal.{u}) : grundyValue (nim o) = o := grundyValue_eq_iff_equiv_nim.2 PGame.equiv_rfl #align pgame.nim_grundy_value SetTheory.PGame.nim_grundyValue theorem grundyValue_eq_iff_equiv (G H : PGame) [G.Impartial] [H.Impartial] : grundyValue G = grundyValue H ↔ (G ≈ H) := grundyValue_eq_iff_equiv_nim.trans (equiv_congr_left.1 (equiv_nim_grundyValue H) _).symm #align pgame.grundy_value_eq_iff_equiv SetTheory.PGame.grundyValue_eq_iff_equiv @[simp] theorem grundyValue_zero : grundyValue 0 = 0 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_zero_equiv) #align pgame.grundy_value_zero SetTheory.PGame.grundyValue_zero theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by rw [← grundyValue_eq_iff_equiv, grundyValue_zero] #align pgame.grundy_value_iff_equiv_zero SetTheory.PGame.grundyValue_iff_equiv_zero @[simp] theorem grundyValue_star : grundyValue star = 1 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_one_equiv) #align pgame.grundy_value_star SetTheory.PGame.grundyValue_star @[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G := by rw [grundyValue_eq_iff_equiv_nim, neg_equiv_iff, neg_nim, ← grundyValue_eq_iff_equiv_nim] #align pgame.grundy_value_neg SetTheory.PGame.grundyValue_neg theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i haveI : (R i).Impartial := @Impartial.moveRight_impartial ⟨l, r, L, R⟩ _ i apply grundyValue_neg #align pgame.grundy_value_eq_mex_right SetTheory.PGame.grundyValue_eq_mex_right -- Todo: this actually generalizes to all ordinals, by defining `Ordinal.lxor` as the pairwise -- `Nat.xor` of base `ω` Cantor normal forms. /-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm
rw [grundyValue_eq_mex_left]
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm
Mathlib.SetTheory.Game.Nim.360_0.mmFMhRYSjViKjcP
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m
Mathlib_SetTheory_Game_Nim
case h.h n : ℕ hn : ∀ m < n, ∀ (m_1 : ℕ), grundyValue (nim ↑m + nim ↑m_1) = ↑(m ^^^ m_1) m : ℕ hm : ∀ m_1 < m, grundyValue (nim ↑n + nim ↑m_1) = ↑(n ^^^ m_1) ⊢ (mex fun i => grundyValue (moveLeft (nim ↑n + nim ↑m) i)) = ↑(n ^^^ m)
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq]; exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h⟩ #align pgame.grundy_value_eq_iff_equiv_nim SetTheory.PGame.grundyValue_eq_iff_equiv_nim @[simp] theorem nim_grundyValue (o : Ordinal.{u}) : grundyValue (nim o) = o := grundyValue_eq_iff_equiv_nim.2 PGame.equiv_rfl #align pgame.nim_grundy_value SetTheory.PGame.nim_grundyValue theorem grundyValue_eq_iff_equiv (G H : PGame) [G.Impartial] [H.Impartial] : grundyValue G = grundyValue H ↔ (G ≈ H) := grundyValue_eq_iff_equiv_nim.trans (equiv_congr_left.1 (equiv_nim_grundyValue H) _).symm #align pgame.grundy_value_eq_iff_equiv SetTheory.PGame.grundyValue_eq_iff_equiv @[simp] theorem grundyValue_zero : grundyValue 0 = 0 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_zero_equiv) #align pgame.grundy_value_zero SetTheory.PGame.grundyValue_zero theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by rw [← grundyValue_eq_iff_equiv, grundyValue_zero] #align pgame.grundy_value_iff_equiv_zero SetTheory.PGame.grundyValue_iff_equiv_zero @[simp] theorem grundyValue_star : grundyValue star = 1 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_one_equiv) #align pgame.grundy_value_star SetTheory.PGame.grundyValue_star @[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G := by rw [grundyValue_eq_iff_equiv_nim, neg_equiv_iff, neg_nim, ← grundyValue_eq_iff_equiv_nim] #align pgame.grundy_value_neg SetTheory.PGame.grundyValue_neg theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i haveI : (R i).Impartial := @Impartial.moveRight_impartial ⟨l, r, L, R⟩ _ i apply grundyValue_neg #align pgame.grundy_value_eq_mex_right SetTheory.PGame.grundyValue_eq_mex_right -- Todo: this actually generalizes to all ordinals, by defining `Ordinal.lxor` as the pairwise -- `Nat.xor` of base `ω` Cantor normal forms. /-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left]
refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_)
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left]
Mathlib.SetTheory.Game.Nim.360_0.mmFMhRYSjViKjcP
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m
Mathlib_SetTheory_Game_Nim
case h.h.refine_1 n : ℕ hn : ∀ m < n, ∀ (m_1 : ℕ), grundyValue (nim ↑m + nim ↑m_1) = ↑(m ^^^ m_1) m : ℕ hm : ∀ m_1 < m, grundyValue (nim ↑n + nim ↑m_1) = ↑(n ^^^ m_1) i : LeftMoves (nim ↑n + nim ↑m) ⊢ grundyValue (moveLeft (nim ↑n + nim ↑m) i) ≠ ↑(n ^^^ m)
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq]; exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h⟩ #align pgame.grundy_value_eq_iff_equiv_nim SetTheory.PGame.grundyValue_eq_iff_equiv_nim @[simp] theorem nim_grundyValue (o : Ordinal.{u}) : grundyValue (nim o) = o := grundyValue_eq_iff_equiv_nim.2 PGame.equiv_rfl #align pgame.nim_grundy_value SetTheory.PGame.nim_grundyValue theorem grundyValue_eq_iff_equiv (G H : PGame) [G.Impartial] [H.Impartial] : grundyValue G = grundyValue H ↔ (G ≈ H) := grundyValue_eq_iff_equiv_nim.trans (equiv_congr_left.1 (equiv_nim_grundyValue H) _).symm #align pgame.grundy_value_eq_iff_equiv SetTheory.PGame.grundyValue_eq_iff_equiv @[simp] theorem grundyValue_zero : grundyValue 0 = 0 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_zero_equiv) #align pgame.grundy_value_zero SetTheory.PGame.grundyValue_zero theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by rw [← grundyValue_eq_iff_equiv, grundyValue_zero] #align pgame.grundy_value_iff_equiv_zero SetTheory.PGame.grundyValue_iff_equiv_zero @[simp] theorem grundyValue_star : grundyValue star = 1 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_one_equiv) #align pgame.grundy_value_star SetTheory.PGame.grundyValue_star @[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G := by rw [grundyValue_eq_iff_equiv_nim, neg_equiv_iff, neg_nim, ← grundyValue_eq_iff_equiv_nim] #align pgame.grundy_value_neg SetTheory.PGame.grundyValue_neg theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i haveI : (R i).Impartial := @Impartial.moveRight_impartial ⟨l, r, L, R⟩ _ i apply grundyValue_neg #align pgame.grundy_value_eq_mex_right SetTheory.PGame.grundyValue_eq_mex_right -- Todo: this actually generalizes to all ordinals, by defining `Ordinal.lxor` as the pairwise -- `Nat.xor` of base `ω` Cantor normal forms. /-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. ·
apply leftMoves_add_cases i
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. ·
Mathlib.SetTheory.Game.Nim.360_0.mmFMhRYSjViKjcP
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m
Mathlib_SetTheory_Game_Nim
case h.h.refine_1.hl n : ℕ hn : ∀ m < n, ∀ (m_1 : ℕ), grundyValue (nim ↑m + nim ↑m_1) = ↑(m ^^^ m_1) m : ℕ hm : ∀ m_1 < m, grundyValue (nim ↑n + nim ↑m_1) = ↑(n ^^^ m_1) i : LeftMoves (nim ↑n + nim ↑m) ⊢ ∀ (i : LeftMoves (nim ↑n)), grundyValue (moveLeft (nim ↑n + nim ↑m) (toLeftMovesAdd (Sum.inl i))) ≠ ↑(n ^^^ m)
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq]; exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h⟩ #align pgame.grundy_value_eq_iff_equiv_nim SetTheory.PGame.grundyValue_eq_iff_equiv_nim @[simp] theorem nim_grundyValue (o : Ordinal.{u}) : grundyValue (nim o) = o := grundyValue_eq_iff_equiv_nim.2 PGame.equiv_rfl #align pgame.nim_grundy_value SetTheory.PGame.nim_grundyValue theorem grundyValue_eq_iff_equiv (G H : PGame) [G.Impartial] [H.Impartial] : grundyValue G = grundyValue H ↔ (G ≈ H) := grundyValue_eq_iff_equiv_nim.trans (equiv_congr_left.1 (equiv_nim_grundyValue H) _).symm #align pgame.grundy_value_eq_iff_equiv SetTheory.PGame.grundyValue_eq_iff_equiv @[simp] theorem grundyValue_zero : grundyValue 0 = 0 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_zero_equiv) #align pgame.grundy_value_zero SetTheory.PGame.grundyValue_zero theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by rw [← grundyValue_eq_iff_equiv, grundyValue_zero] #align pgame.grundy_value_iff_equiv_zero SetTheory.PGame.grundyValue_iff_equiv_zero @[simp] theorem grundyValue_star : grundyValue star = 1 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_one_equiv) #align pgame.grundy_value_star SetTheory.PGame.grundyValue_star @[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G := by rw [grundyValue_eq_iff_equiv_nim, neg_equiv_iff, neg_nim, ← grundyValue_eq_iff_equiv_nim] #align pgame.grundy_value_neg SetTheory.PGame.grundyValue_neg theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i haveI : (R i).Impartial := @Impartial.moveRight_impartial ⟨l, r, L, R⟩ _ i apply grundyValue_neg #align pgame.grundy_value_eq_mex_right SetTheory.PGame.grundyValue_eq_mex_right -- Todo: this actually generalizes to all ordinals, by defining `Ordinal.lxor` as the pairwise -- `Nat.xor` of base `ω` Cantor normal forms. /-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`.
refine' fun a => leftMovesNimRecOn a fun ok hk => _
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`.
Mathlib.SetTheory.Game.Nim.360_0.mmFMhRYSjViKjcP
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m
Mathlib_SetTheory_Game_Nim
case h.h.refine_1.hl n : ℕ hn : ∀ m < n, ∀ (m_1 : ℕ), grundyValue (nim ↑m + nim ↑m_1) = ↑(m ^^^ m_1) m : ℕ hm : ∀ m_1 < m, grundyValue (nim ↑n + nim ↑m_1) = ↑(n ^^^ m_1) i : LeftMoves (nim ↑n + nim ↑m) a : LeftMoves (nim ↑n) ok : Ordinal.{u} hk : ok < ↑n ⊢ grundyValue (moveLeft (nim ↑n + nim ↑m) (toLeftMovesAdd (Sum.inl (toLeftMovesNim { val := ok, property := hk })))) ≠ ↑(n ^^^ m)
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq]; exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h⟩ #align pgame.grundy_value_eq_iff_equiv_nim SetTheory.PGame.grundyValue_eq_iff_equiv_nim @[simp] theorem nim_grundyValue (o : Ordinal.{u}) : grundyValue (nim o) = o := grundyValue_eq_iff_equiv_nim.2 PGame.equiv_rfl #align pgame.nim_grundy_value SetTheory.PGame.nim_grundyValue theorem grundyValue_eq_iff_equiv (G H : PGame) [G.Impartial] [H.Impartial] : grundyValue G = grundyValue H ↔ (G ≈ H) := grundyValue_eq_iff_equiv_nim.trans (equiv_congr_left.1 (equiv_nim_grundyValue H) _).symm #align pgame.grundy_value_eq_iff_equiv SetTheory.PGame.grundyValue_eq_iff_equiv @[simp] theorem grundyValue_zero : grundyValue 0 = 0 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_zero_equiv) #align pgame.grundy_value_zero SetTheory.PGame.grundyValue_zero theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by rw [← grundyValue_eq_iff_equiv, grundyValue_zero] #align pgame.grundy_value_iff_equiv_zero SetTheory.PGame.grundyValue_iff_equiv_zero @[simp] theorem grundyValue_star : grundyValue star = 1 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_one_equiv) #align pgame.grundy_value_star SetTheory.PGame.grundyValue_star @[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G := by rw [grundyValue_eq_iff_equiv_nim, neg_equiv_iff, neg_nim, ← grundyValue_eq_iff_equiv_nim] #align pgame.grundy_value_neg SetTheory.PGame.grundyValue_neg theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i haveI : (R i).Impartial := @Impartial.moveRight_impartial ⟨l, r, L, R⟩ _ i apply grundyValue_neg #align pgame.grundy_value_eq_mex_right SetTheory.PGame.grundyValue_eq_mex_right -- Todo: this actually generalizes to all ordinals, by defining `Ordinal.lxor` as the pairwise -- `Nat.xor` of base `ω` Cantor normal forms. /-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _
obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _))
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _
Mathlib.SetTheory.Game.Nim.360_0.mmFMhRYSjViKjcP
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m
Mathlib_SetTheory_Game_Nim
case h.h.refine_1.hl.intro n : ℕ hn : ∀ m < n, ∀ (m_1 : ℕ), grundyValue (nim ↑m + nim ↑m_1) = ↑(m ^^^ m_1) m : ℕ hm : ∀ m_1 < m, grundyValue (nim ↑n + nim ↑m_1) = ↑(n ^^^ m_1) i : LeftMoves (nim ↑n + nim ↑m) a : LeftMoves (nim ↑n) k : ℕ hk : ↑k < ↑n ⊢ grundyValue (moveLeft (nim ↑n + nim ↑m) (toLeftMovesAdd (Sum.inl (toLeftMovesNim { val := ↑k, property := hk })))) ≠ ↑(n ^^^ m)
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq]; exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h⟩ #align pgame.grundy_value_eq_iff_equiv_nim SetTheory.PGame.grundyValue_eq_iff_equiv_nim @[simp] theorem nim_grundyValue (o : Ordinal.{u}) : grundyValue (nim o) = o := grundyValue_eq_iff_equiv_nim.2 PGame.equiv_rfl #align pgame.nim_grundy_value SetTheory.PGame.nim_grundyValue theorem grundyValue_eq_iff_equiv (G H : PGame) [G.Impartial] [H.Impartial] : grundyValue G = grundyValue H ↔ (G ≈ H) := grundyValue_eq_iff_equiv_nim.trans (equiv_congr_left.1 (equiv_nim_grundyValue H) _).symm #align pgame.grundy_value_eq_iff_equiv SetTheory.PGame.grundyValue_eq_iff_equiv @[simp] theorem grundyValue_zero : grundyValue 0 = 0 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_zero_equiv) #align pgame.grundy_value_zero SetTheory.PGame.grundyValue_zero theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by rw [← grundyValue_eq_iff_equiv, grundyValue_zero] #align pgame.grundy_value_iff_equiv_zero SetTheory.PGame.grundyValue_iff_equiv_zero @[simp] theorem grundyValue_star : grundyValue star = 1 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_one_equiv) #align pgame.grundy_value_star SetTheory.PGame.grundyValue_star @[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G := by rw [grundyValue_eq_iff_equiv_nim, neg_equiv_iff, neg_nim, ← grundyValue_eq_iff_equiv_nim] #align pgame.grundy_value_neg SetTheory.PGame.grundyValue_neg theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i haveI : (R i).Impartial := @Impartial.moveRight_impartial ⟨l, r, L, R⟩ _ i apply grundyValue_neg #align pgame.grundy_value_eq_mex_right SetTheory.PGame.grundyValue_eq_mex_right -- Todo: this actually generalizes to all ordinals, by defining `Ordinal.lxor` as the pairwise -- `Nat.xor` of base `ω` Cantor normal forms. /-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _))
simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply]
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _))
Mathlib.SetTheory.Game.Nim.360_0.mmFMhRYSjViKjcP
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m
Mathlib_SetTheory_Game_Nim
case h.h.refine_1.hl.intro n : ℕ hn : ∀ m < n, ∀ (m_1 : ℕ), grundyValue (nim ↑m + nim ↑m_1) = ↑(m ^^^ m_1) m : ℕ hm : ∀ m_1 < m, grundyValue (nim ↑n + nim ↑m_1) = ↑(n ^^^ m_1) i : LeftMoves (nim ↑n + nim ↑m) a : LeftMoves (nim ↑n) k : ℕ hk : ↑k < ↑n ⊢ grundyValue (nim ↑k + nim ↑m) ≠ ↑(n ^^^ m)
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq]; exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h⟩ #align pgame.grundy_value_eq_iff_equiv_nim SetTheory.PGame.grundyValue_eq_iff_equiv_nim @[simp] theorem nim_grundyValue (o : Ordinal.{u}) : grundyValue (nim o) = o := grundyValue_eq_iff_equiv_nim.2 PGame.equiv_rfl #align pgame.nim_grundy_value SetTheory.PGame.nim_grundyValue theorem grundyValue_eq_iff_equiv (G H : PGame) [G.Impartial] [H.Impartial] : grundyValue G = grundyValue H ↔ (G ≈ H) := grundyValue_eq_iff_equiv_nim.trans (equiv_congr_left.1 (equiv_nim_grundyValue H) _).symm #align pgame.grundy_value_eq_iff_equiv SetTheory.PGame.grundyValue_eq_iff_equiv @[simp] theorem grundyValue_zero : grundyValue 0 = 0 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_zero_equiv) #align pgame.grundy_value_zero SetTheory.PGame.grundyValue_zero theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by rw [← grundyValue_eq_iff_equiv, grundyValue_zero] #align pgame.grundy_value_iff_equiv_zero SetTheory.PGame.grundyValue_iff_equiv_zero @[simp] theorem grundyValue_star : grundyValue star = 1 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_one_equiv) #align pgame.grundy_value_star SetTheory.PGame.grundyValue_star @[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G := by rw [grundyValue_eq_iff_equiv_nim, neg_equiv_iff, neg_nim, ← grundyValue_eq_iff_equiv_nim] #align pgame.grundy_value_neg SetTheory.PGame.grundyValue_neg theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i haveI : (R i).Impartial := @Impartial.moveRight_impartial ⟨l, r, L, R⟩ _ i apply grundyValue_neg #align pgame.grundy_value_eq_mex_right SetTheory.PGame.grundyValue_eq_mex_right -- Todo: this actually generalizes to all ordinals, by defining `Ordinal.lxor` as the pairwise -- `Nat.xor` of base `ω` Cantor normal forms. /-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity.
rw [nat_cast_lt] at hk
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity.
Mathlib.SetTheory.Game.Nim.360_0.mmFMhRYSjViKjcP
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m
Mathlib_SetTheory_Game_Nim
case h.h.refine_1.hl.intro n : ℕ hn : ∀ m < n, ∀ (m_1 : ℕ), grundyValue (nim ↑m + nim ↑m_1) = ↑(m ^^^ m_1) m : ℕ hm : ∀ m_1 < m, grundyValue (nim ↑n + nim ↑m_1) = ↑(n ^^^ m_1) i : LeftMoves (nim ↑n + nim ↑m) a : LeftMoves (nim ↑n) k : ℕ hk : k < n ⊢ grundyValue (nim ↑k + nim ↑m) ≠ ↑(n ^^^ m)
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq]; exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h⟩ #align pgame.grundy_value_eq_iff_equiv_nim SetTheory.PGame.grundyValue_eq_iff_equiv_nim @[simp] theorem nim_grundyValue (o : Ordinal.{u}) : grundyValue (nim o) = o := grundyValue_eq_iff_equiv_nim.2 PGame.equiv_rfl #align pgame.nim_grundy_value SetTheory.PGame.nim_grundyValue theorem grundyValue_eq_iff_equiv (G H : PGame) [G.Impartial] [H.Impartial] : grundyValue G = grundyValue H ↔ (G ≈ H) := grundyValue_eq_iff_equiv_nim.trans (equiv_congr_left.1 (equiv_nim_grundyValue H) _).symm #align pgame.grundy_value_eq_iff_equiv SetTheory.PGame.grundyValue_eq_iff_equiv @[simp] theorem grundyValue_zero : grundyValue 0 = 0 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_zero_equiv) #align pgame.grundy_value_zero SetTheory.PGame.grundyValue_zero theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by rw [← grundyValue_eq_iff_equiv, grundyValue_zero] #align pgame.grundy_value_iff_equiv_zero SetTheory.PGame.grundyValue_iff_equiv_zero @[simp] theorem grundyValue_star : grundyValue star = 1 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_one_equiv) #align pgame.grundy_value_star SetTheory.PGame.grundyValue_star @[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G := by rw [grundyValue_eq_iff_equiv_nim, neg_equiv_iff, neg_nim, ← grundyValue_eq_iff_equiv_nim] #align pgame.grundy_value_neg SetTheory.PGame.grundyValue_neg theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i haveI : (R i).Impartial := @Impartial.moveRight_impartial ⟨l, r, L, R⟩ _ i apply grundyValue_neg #align pgame.grundy_value_eq_mex_right SetTheory.PGame.grundyValue_eq_mex_right -- Todo: this actually generalizes to all ordinals, by defining `Ordinal.lxor` as the pairwise -- `Nat.xor` of base `ω` Cantor normal forms. /-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk
first | rw [hn _ hk] | rw [hm _ hk]
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk
Mathlib.SetTheory.Game.Nim.360_0.mmFMhRYSjViKjcP
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m
Mathlib_SetTheory_Game_Nim
case h.h.refine_1.hl.intro n : ℕ hn : ∀ m < n, ∀ (m_1 : ℕ), grundyValue (nim ↑m + nim ↑m_1) = ↑(m ^^^ m_1) m : ℕ hm : ∀ m_1 < m, grundyValue (nim ↑n + nim ↑m_1) = ↑(n ^^^ m_1) i : LeftMoves (nim ↑n + nim ↑m) a : LeftMoves (nim ↑n) k : ℕ hk : k < n ⊢ grundyValue (nim ↑k + nim ↑m) ≠ ↑(n ^^^ m)
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq]; exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h⟩ #align pgame.grundy_value_eq_iff_equiv_nim SetTheory.PGame.grundyValue_eq_iff_equiv_nim @[simp] theorem nim_grundyValue (o : Ordinal.{u}) : grundyValue (nim o) = o := grundyValue_eq_iff_equiv_nim.2 PGame.equiv_rfl #align pgame.nim_grundy_value SetTheory.PGame.nim_grundyValue theorem grundyValue_eq_iff_equiv (G H : PGame) [G.Impartial] [H.Impartial] : grundyValue G = grundyValue H ↔ (G ≈ H) := grundyValue_eq_iff_equiv_nim.trans (equiv_congr_left.1 (equiv_nim_grundyValue H) _).symm #align pgame.grundy_value_eq_iff_equiv SetTheory.PGame.grundyValue_eq_iff_equiv @[simp] theorem grundyValue_zero : grundyValue 0 = 0 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_zero_equiv) #align pgame.grundy_value_zero SetTheory.PGame.grundyValue_zero theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by rw [← grundyValue_eq_iff_equiv, grundyValue_zero] #align pgame.grundy_value_iff_equiv_zero SetTheory.PGame.grundyValue_iff_equiv_zero @[simp] theorem grundyValue_star : grundyValue star = 1 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_one_equiv) #align pgame.grundy_value_star SetTheory.PGame.grundyValue_star @[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G := by rw [grundyValue_eq_iff_equiv_nim, neg_equiv_iff, neg_nim, ← grundyValue_eq_iff_equiv_nim] #align pgame.grundy_value_neg SetTheory.PGame.grundyValue_neg theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i haveI : (R i).Impartial := @Impartial.moveRight_impartial ⟨l, r, L, R⟩ _ i apply grundyValue_neg #align pgame.grundy_value_eq_mex_right SetTheory.PGame.grundyValue_eq_mex_right -- Todo: this actually generalizes to all ordinals, by defining `Ordinal.lxor` as the pairwise -- `Nat.xor` of base `ω` Cantor normal forms. /-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk first |
rw [hn _ hk]
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk first |
Mathlib.SetTheory.Game.Nim.360_0.mmFMhRYSjViKjcP
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m
Mathlib_SetTheory_Game_Nim
case h.h.refine_1.hl.intro n : ℕ hn : ∀ m < n, ∀ (m_1 : ℕ), grundyValue (nim ↑m + nim ↑m_1) = ↑(m ^^^ m_1) m : ℕ hm : ∀ m_1 < m, grundyValue (nim ↑n + nim ↑m_1) = ↑(n ^^^ m_1) i : LeftMoves (nim ↑n + nim ↑m) a : LeftMoves (nim ↑n) k : ℕ hk : k < n ⊢ ↑(k ^^^ m) ≠ ↑(n ^^^ m)
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq]; exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h⟩ #align pgame.grundy_value_eq_iff_equiv_nim SetTheory.PGame.grundyValue_eq_iff_equiv_nim @[simp] theorem nim_grundyValue (o : Ordinal.{u}) : grundyValue (nim o) = o := grundyValue_eq_iff_equiv_nim.2 PGame.equiv_rfl #align pgame.nim_grundy_value SetTheory.PGame.nim_grundyValue theorem grundyValue_eq_iff_equiv (G H : PGame) [G.Impartial] [H.Impartial] : grundyValue G = grundyValue H ↔ (G ≈ H) := grundyValue_eq_iff_equiv_nim.trans (equiv_congr_left.1 (equiv_nim_grundyValue H) _).symm #align pgame.grundy_value_eq_iff_equiv SetTheory.PGame.grundyValue_eq_iff_equiv @[simp] theorem grundyValue_zero : grundyValue 0 = 0 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_zero_equiv) #align pgame.grundy_value_zero SetTheory.PGame.grundyValue_zero theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by rw [← grundyValue_eq_iff_equiv, grundyValue_zero] #align pgame.grundy_value_iff_equiv_zero SetTheory.PGame.grundyValue_iff_equiv_zero @[simp] theorem grundyValue_star : grundyValue star = 1 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_one_equiv) #align pgame.grundy_value_star SetTheory.PGame.grundyValue_star @[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G := by rw [grundyValue_eq_iff_equiv_nim, neg_equiv_iff, neg_nim, ← grundyValue_eq_iff_equiv_nim] #align pgame.grundy_value_neg SetTheory.PGame.grundyValue_neg theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i haveI : (R i).Impartial := @Impartial.moveRight_impartial ⟨l, r, L, R⟩ _ i apply grundyValue_neg #align pgame.grundy_value_eq_mex_right SetTheory.PGame.grundyValue_eq_mex_right -- Todo: this actually generalizes to all ordinals, by defining `Ordinal.lxor` as the pairwise -- `Nat.xor` of base `ω` Cantor normal forms. /-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk first | rw [hn _ hk] | rw [hm _ hk]
refine' fun h => hk.ne _
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk first | rw [hn _ hk] | rw [hm _ hk]
Mathlib.SetTheory.Game.Nim.360_0.mmFMhRYSjViKjcP
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m
Mathlib_SetTheory_Game_Nim
case h.h.refine_1.hl.intro n : ℕ hn : ∀ m < n, ∀ (m_1 : ℕ), grundyValue (nim ↑m + nim ↑m_1) = ↑(m ^^^ m_1) m : ℕ hm : ∀ m_1 < m, grundyValue (nim ↑n + nim ↑m_1) = ↑(n ^^^ m_1) i : LeftMoves (nim ↑n + nim ↑m) a : LeftMoves (nim ↑n) k : ℕ hk : k < n h : ↑(k ^^^ m) = ↑(n ^^^ m) ⊢ k = n
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq]; exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h⟩ #align pgame.grundy_value_eq_iff_equiv_nim SetTheory.PGame.grundyValue_eq_iff_equiv_nim @[simp] theorem nim_grundyValue (o : Ordinal.{u}) : grundyValue (nim o) = o := grundyValue_eq_iff_equiv_nim.2 PGame.equiv_rfl #align pgame.nim_grundy_value SetTheory.PGame.nim_grundyValue theorem grundyValue_eq_iff_equiv (G H : PGame) [G.Impartial] [H.Impartial] : grundyValue G = grundyValue H ↔ (G ≈ H) := grundyValue_eq_iff_equiv_nim.trans (equiv_congr_left.1 (equiv_nim_grundyValue H) _).symm #align pgame.grundy_value_eq_iff_equiv SetTheory.PGame.grundyValue_eq_iff_equiv @[simp] theorem grundyValue_zero : grundyValue 0 = 0 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_zero_equiv) #align pgame.grundy_value_zero SetTheory.PGame.grundyValue_zero theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by rw [← grundyValue_eq_iff_equiv, grundyValue_zero] #align pgame.grundy_value_iff_equiv_zero SetTheory.PGame.grundyValue_iff_equiv_zero @[simp] theorem grundyValue_star : grundyValue star = 1 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_one_equiv) #align pgame.grundy_value_star SetTheory.PGame.grundyValue_star @[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G := by rw [grundyValue_eq_iff_equiv_nim, neg_equiv_iff, neg_nim, ← grundyValue_eq_iff_equiv_nim] #align pgame.grundy_value_neg SetTheory.PGame.grundyValue_neg theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i haveI : (R i).Impartial := @Impartial.moveRight_impartial ⟨l, r, L, R⟩ _ i apply grundyValue_neg #align pgame.grundy_value_eq_mex_right SetTheory.PGame.grundyValue_eq_mex_right -- Todo: this actually generalizes to all ordinals, by defining `Ordinal.lxor` as the pairwise -- `Nat.xor` of base `ω` Cantor normal forms. /-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk first | rw [hn _ hk] | rw [hm _ hk] refine' fun h => hk.ne _
rw [Ordinal.nat_cast_inj] at h
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk first | rw [hn _ hk] | rw [hm _ hk] refine' fun h => hk.ne _
Mathlib.SetTheory.Game.Nim.360_0.mmFMhRYSjViKjcP
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m
Mathlib_SetTheory_Game_Nim
case h.h.refine_1.hl.intro n : ℕ hn : ∀ m < n, ∀ (m_1 : ℕ), grundyValue (nim ↑m + nim ↑m_1) = ↑(m ^^^ m_1) m : ℕ hm : ∀ m_1 < m, grundyValue (nim ↑n + nim ↑m_1) = ↑(n ^^^ m_1) i : LeftMoves (nim ↑n + nim ↑m) a : LeftMoves (nim ↑n) k : ℕ hk : k < n h : k ^^^ m = n ^^^ m ⊢ k = n
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq]; exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h⟩ #align pgame.grundy_value_eq_iff_equiv_nim SetTheory.PGame.grundyValue_eq_iff_equiv_nim @[simp] theorem nim_grundyValue (o : Ordinal.{u}) : grundyValue (nim o) = o := grundyValue_eq_iff_equiv_nim.2 PGame.equiv_rfl #align pgame.nim_grundy_value SetTheory.PGame.nim_grundyValue theorem grundyValue_eq_iff_equiv (G H : PGame) [G.Impartial] [H.Impartial] : grundyValue G = grundyValue H ↔ (G ≈ H) := grundyValue_eq_iff_equiv_nim.trans (equiv_congr_left.1 (equiv_nim_grundyValue H) _).symm #align pgame.grundy_value_eq_iff_equiv SetTheory.PGame.grundyValue_eq_iff_equiv @[simp] theorem grundyValue_zero : grundyValue 0 = 0 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_zero_equiv) #align pgame.grundy_value_zero SetTheory.PGame.grundyValue_zero theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by rw [← grundyValue_eq_iff_equiv, grundyValue_zero] #align pgame.grundy_value_iff_equiv_zero SetTheory.PGame.grundyValue_iff_equiv_zero @[simp] theorem grundyValue_star : grundyValue star = 1 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_one_equiv) #align pgame.grundy_value_star SetTheory.PGame.grundyValue_star @[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G := by rw [grundyValue_eq_iff_equiv_nim, neg_equiv_iff, neg_nim, ← grundyValue_eq_iff_equiv_nim] #align pgame.grundy_value_neg SetTheory.PGame.grundyValue_neg theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i haveI : (R i).Impartial := @Impartial.moveRight_impartial ⟨l, r, L, R⟩ _ i apply grundyValue_neg #align pgame.grundy_value_eq_mex_right SetTheory.PGame.grundyValue_eq_mex_right -- Todo: this actually generalizes to all ordinals, by defining `Ordinal.lxor` as the pairwise -- `Nat.xor` of base `ω` Cantor normal forms. /-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk first | rw [hn _ hk] | rw [hm _ hk] refine' fun h => hk.ne _ rw [Ordinal.nat_cast_inj] at h
first | rwa [Nat.xor_left_inj] at h | rwa [Nat.xor_right_inj] at h
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk first | rw [hn _ hk] | rw [hm _ hk] refine' fun h => hk.ne _ rw [Ordinal.nat_cast_inj] at h
Mathlib.SetTheory.Game.Nim.360_0.mmFMhRYSjViKjcP
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m
Mathlib_SetTheory_Game_Nim
case h.h.refine_1.hl.intro n : ℕ hn : ∀ m < n, ∀ (m_1 : ℕ), grundyValue (nim ↑m + nim ↑m_1) = ↑(m ^^^ m_1) m : ℕ hm : ∀ m_1 < m, grundyValue (nim ↑n + nim ↑m_1) = ↑(n ^^^ m_1) i : LeftMoves (nim ↑n + nim ↑m) a : LeftMoves (nim ↑n) k : ℕ hk : k < n h : k ^^^ m = n ^^^ m ⊢ k = n
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq]; exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h⟩ #align pgame.grundy_value_eq_iff_equiv_nim SetTheory.PGame.grundyValue_eq_iff_equiv_nim @[simp] theorem nim_grundyValue (o : Ordinal.{u}) : grundyValue (nim o) = o := grundyValue_eq_iff_equiv_nim.2 PGame.equiv_rfl #align pgame.nim_grundy_value SetTheory.PGame.nim_grundyValue theorem grundyValue_eq_iff_equiv (G H : PGame) [G.Impartial] [H.Impartial] : grundyValue G = grundyValue H ↔ (G ≈ H) := grundyValue_eq_iff_equiv_nim.trans (equiv_congr_left.1 (equiv_nim_grundyValue H) _).symm #align pgame.grundy_value_eq_iff_equiv SetTheory.PGame.grundyValue_eq_iff_equiv @[simp] theorem grundyValue_zero : grundyValue 0 = 0 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_zero_equiv) #align pgame.grundy_value_zero SetTheory.PGame.grundyValue_zero theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by rw [← grundyValue_eq_iff_equiv, grundyValue_zero] #align pgame.grundy_value_iff_equiv_zero SetTheory.PGame.grundyValue_iff_equiv_zero @[simp] theorem grundyValue_star : grundyValue star = 1 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_one_equiv) #align pgame.grundy_value_star SetTheory.PGame.grundyValue_star @[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G := by rw [grundyValue_eq_iff_equiv_nim, neg_equiv_iff, neg_nim, ← grundyValue_eq_iff_equiv_nim] #align pgame.grundy_value_neg SetTheory.PGame.grundyValue_neg theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i haveI : (R i).Impartial := @Impartial.moveRight_impartial ⟨l, r, L, R⟩ _ i apply grundyValue_neg #align pgame.grundy_value_eq_mex_right SetTheory.PGame.grundyValue_eq_mex_right -- Todo: this actually generalizes to all ordinals, by defining `Ordinal.lxor` as the pairwise -- `Nat.xor` of base `ω` Cantor normal forms. /-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk first | rw [hn _ hk] | rw [hm _ hk] refine' fun h => hk.ne _ rw [Ordinal.nat_cast_inj] at h first |
rwa [Nat.xor_left_inj] at h
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk first | rw [hn _ hk] | rw [hm _ hk] refine' fun h => hk.ne _ rw [Ordinal.nat_cast_inj] at h first |
Mathlib.SetTheory.Game.Nim.360_0.mmFMhRYSjViKjcP
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m
Mathlib_SetTheory_Game_Nim
case h.h.refine_1.hr n : ℕ hn : ∀ m < n, ∀ (m_1 : ℕ), grundyValue (nim ↑m + nim ↑m_1) = ↑(m ^^^ m_1) m : ℕ hm : ∀ m_1 < m, grundyValue (nim ↑n + nim ↑m_1) = ↑(n ^^^ m_1) i : LeftMoves (nim ↑n + nim ↑m) ⊢ ∀ (i : LeftMoves (nim ↑m)), grundyValue (moveLeft (nim ↑n + nim ↑m) (toLeftMovesAdd (Sum.inr i))) ≠ ↑(n ^^^ m)
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq]; exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h⟩ #align pgame.grundy_value_eq_iff_equiv_nim SetTheory.PGame.grundyValue_eq_iff_equiv_nim @[simp] theorem nim_grundyValue (o : Ordinal.{u}) : grundyValue (nim o) = o := grundyValue_eq_iff_equiv_nim.2 PGame.equiv_rfl #align pgame.nim_grundy_value SetTheory.PGame.nim_grundyValue theorem grundyValue_eq_iff_equiv (G H : PGame) [G.Impartial] [H.Impartial] : grundyValue G = grundyValue H ↔ (G ≈ H) := grundyValue_eq_iff_equiv_nim.trans (equiv_congr_left.1 (equiv_nim_grundyValue H) _).symm #align pgame.grundy_value_eq_iff_equiv SetTheory.PGame.grundyValue_eq_iff_equiv @[simp] theorem grundyValue_zero : grundyValue 0 = 0 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_zero_equiv) #align pgame.grundy_value_zero SetTheory.PGame.grundyValue_zero theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by rw [← grundyValue_eq_iff_equiv, grundyValue_zero] #align pgame.grundy_value_iff_equiv_zero SetTheory.PGame.grundyValue_iff_equiv_zero @[simp] theorem grundyValue_star : grundyValue star = 1 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_one_equiv) #align pgame.grundy_value_star SetTheory.PGame.grundyValue_star @[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G := by rw [grundyValue_eq_iff_equiv_nim, neg_equiv_iff, neg_nim, ← grundyValue_eq_iff_equiv_nim] #align pgame.grundy_value_neg SetTheory.PGame.grundyValue_neg theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i haveI : (R i).Impartial := @Impartial.moveRight_impartial ⟨l, r, L, R⟩ _ i apply grundyValue_neg #align pgame.grundy_value_eq_mex_right SetTheory.PGame.grundyValue_eq_mex_right -- Todo: this actually generalizes to all ordinals, by defining `Ordinal.lxor` as the pairwise -- `Nat.xor` of base `ω` Cantor normal forms. /-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`.
refine' fun a => leftMovesNimRecOn a fun ok hk => _
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`.
Mathlib.SetTheory.Game.Nim.360_0.mmFMhRYSjViKjcP
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m
Mathlib_SetTheory_Game_Nim
case h.h.refine_1.hr n : ℕ hn : ∀ m < n, ∀ (m_1 : ℕ), grundyValue (nim ↑m + nim ↑m_1) = ↑(m ^^^ m_1) m : ℕ hm : ∀ m_1 < m, grundyValue (nim ↑n + nim ↑m_1) = ↑(n ^^^ m_1) i : LeftMoves (nim ↑n + nim ↑m) a : LeftMoves (nim ↑m) ok : Ordinal.{u} hk : ok < ↑m ⊢ grundyValue (moveLeft (nim ↑n + nim ↑m) (toLeftMovesAdd (Sum.inr (toLeftMovesNim { val := ok, property := hk })))) ≠ ↑(n ^^^ m)
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq]; exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h⟩ #align pgame.grundy_value_eq_iff_equiv_nim SetTheory.PGame.grundyValue_eq_iff_equiv_nim @[simp] theorem nim_grundyValue (o : Ordinal.{u}) : grundyValue (nim o) = o := grundyValue_eq_iff_equiv_nim.2 PGame.equiv_rfl #align pgame.nim_grundy_value SetTheory.PGame.nim_grundyValue theorem grundyValue_eq_iff_equiv (G H : PGame) [G.Impartial] [H.Impartial] : grundyValue G = grundyValue H ↔ (G ≈ H) := grundyValue_eq_iff_equiv_nim.trans (equiv_congr_left.1 (equiv_nim_grundyValue H) _).symm #align pgame.grundy_value_eq_iff_equiv SetTheory.PGame.grundyValue_eq_iff_equiv @[simp] theorem grundyValue_zero : grundyValue 0 = 0 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_zero_equiv) #align pgame.grundy_value_zero SetTheory.PGame.grundyValue_zero theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by rw [← grundyValue_eq_iff_equiv, grundyValue_zero] #align pgame.grundy_value_iff_equiv_zero SetTheory.PGame.grundyValue_iff_equiv_zero @[simp] theorem grundyValue_star : grundyValue star = 1 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_one_equiv) #align pgame.grundy_value_star SetTheory.PGame.grundyValue_star @[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G := by rw [grundyValue_eq_iff_equiv_nim, neg_equiv_iff, neg_nim, ← grundyValue_eq_iff_equiv_nim] #align pgame.grundy_value_neg SetTheory.PGame.grundyValue_neg theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i haveI : (R i).Impartial := @Impartial.moveRight_impartial ⟨l, r, L, R⟩ _ i apply grundyValue_neg #align pgame.grundy_value_eq_mex_right SetTheory.PGame.grundyValue_eq_mex_right -- Todo: this actually generalizes to all ordinals, by defining `Ordinal.lxor` as the pairwise -- `Nat.xor` of base `ω` Cantor normal forms. /-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _
obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _))
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _
Mathlib.SetTheory.Game.Nim.360_0.mmFMhRYSjViKjcP
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m
Mathlib_SetTheory_Game_Nim
case h.h.refine_1.hr.intro n : ℕ hn : ∀ m < n, ∀ (m_1 : ℕ), grundyValue (nim ↑m + nim ↑m_1) = ↑(m ^^^ m_1) m : ℕ hm : ∀ m_1 < m, grundyValue (nim ↑n + nim ↑m_1) = ↑(n ^^^ m_1) i : LeftMoves (nim ↑n + nim ↑m) a : LeftMoves (nim ↑m) k : ℕ hk : ↑k < ↑m ⊢ grundyValue (moveLeft (nim ↑n + nim ↑m) (toLeftMovesAdd (Sum.inr (toLeftMovesNim { val := ↑k, property := hk })))) ≠ ↑(n ^^^ m)
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq]; exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h⟩ #align pgame.grundy_value_eq_iff_equiv_nim SetTheory.PGame.grundyValue_eq_iff_equiv_nim @[simp] theorem nim_grundyValue (o : Ordinal.{u}) : grundyValue (nim o) = o := grundyValue_eq_iff_equiv_nim.2 PGame.equiv_rfl #align pgame.nim_grundy_value SetTheory.PGame.nim_grundyValue theorem grundyValue_eq_iff_equiv (G H : PGame) [G.Impartial] [H.Impartial] : grundyValue G = grundyValue H ↔ (G ≈ H) := grundyValue_eq_iff_equiv_nim.trans (equiv_congr_left.1 (equiv_nim_grundyValue H) _).symm #align pgame.grundy_value_eq_iff_equiv SetTheory.PGame.grundyValue_eq_iff_equiv @[simp] theorem grundyValue_zero : grundyValue 0 = 0 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_zero_equiv) #align pgame.grundy_value_zero SetTheory.PGame.grundyValue_zero theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by rw [← grundyValue_eq_iff_equiv, grundyValue_zero] #align pgame.grundy_value_iff_equiv_zero SetTheory.PGame.grundyValue_iff_equiv_zero @[simp] theorem grundyValue_star : grundyValue star = 1 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_one_equiv) #align pgame.grundy_value_star SetTheory.PGame.grundyValue_star @[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G := by rw [grundyValue_eq_iff_equiv_nim, neg_equiv_iff, neg_nim, ← grundyValue_eq_iff_equiv_nim] #align pgame.grundy_value_neg SetTheory.PGame.grundyValue_neg theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i haveI : (R i).Impartial := @Impartial.moveRight_impartial ⟨l, r, L, R⟩ _ i apply grundyValue_neg #align pgame.grundy_value_eq_mex_right SetTheory.PGame.grundyValue_eq_mex_right -- Todo: this actually generalizes to all ordinals, by defining `Ordinal.lxor` as the pairwise -- `Nat.xor` of base `ω` Cantor normal forms. /-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _))
simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply]
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _))
Mathlib.SetTheory.Game.Nim.360_0.mmFMhRYSjViKjcP
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m
Mathlib_SetTheory_Game_Nim
case h.h.refine_1.hr.intro n : ℕ hn : ∀ m < n, ∀ (m_1 : ℕ), grundyValue (nim ↑m + nim ↑m_1) = ↑(m ^^^ m_1) m : ℕ hm : ∀ m_1 < m, grundyValue (nim ↑n + nim ↑m_1) = ↑(n ^^^ m_1) i : LeftMoves (nim ↑n + nim ↑m) a : LeftMoves (nim ↑m) k : ℕ hk : ↑k < ↑m ⊢ grundyValue (nim ↑n + nim ↑k) ≠ ↑(n ^^^ m)
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq]; exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h⟩ #align pgame.grundy_value_eq_iff_equiv_nim SetTheory.PGame.grundyValue_eq_iff_equiv_nim @[simp] theorem nim_grundyValue (o : Ordinal.{u}) : grundyValue (nim o) = o := grundyValue_eq_iff_equiv_nim.2 PGame.equiv_rfl #align pgame.nim_grundy_value SetTheory.PGame.nim_grundyValue theorem grundyValue_eq_iff_equiv (G H : PGame) [G.Impartial] [H.Impartial] : grundyValue G = grundyValue H ↔ (G ≈ H) := grundyValue_eq_iff_equiv_nim.trans (equiv_congr_left.1 (equiv_nim_grundyValue H) _).symm #align pgame.grundy_value_eq_iff_equiv SetTheory.PGame.grundyValue_eq_iff_equiv @[simp] theorem grundyValue_zero : grundyValue 0 = 0 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_zero_equiv) #align pgame.grundy_value_zero SetTheory.PGame.grundyValue_zero theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by rw [← grundyValue_eq_iff_equiv, grundyValue_zero] #align pgame.grundy_value_iff_equiv_zero SetTheory.PGame.grundyValue_iff_equiv_zero @[simp] theorem grundyValue_star : grundyValue star = 1 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_one_equiv) #align pgame.grundy_value_star SetTheory.PGame.grundyValue_star @[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G := by rw [grundyValue_eq_iff_equiv_nim, neg_equiv_iff, neg_nim, ← grundyValue_eq_iff_equiv_nim] #align pgame.grundy_value_neg SetTheory.PGame.grundyValue_neg theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i haveI : (R i).Impartial := @Impartial.moveRight_impartial ⟨l, r, L, R⟩ _ i apply grundyValue_neg #align pgame.grundy_value_eq_mex_right SetTheory.PGame.grundyValue_eq_mex_right -- Todo: this actually generalizes to all ordinals, by defining `Ordinal.lxor` as the pairwise -- `Nat.xor` of base `ω` Cantor normal forms. /-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity.
rw [nat_cast_lt] at hk
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity.
Mathlib.SetTheory.Game.Nim.360_0.mmFMhRYSjViKjcP
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m
Mathlib_SetTheory_Game_Nim
case h.h.refine_1.hr.intro n : ℕ hn : ∀ m < n, ∀ (m_1 : ℕ), grundyValue (nim ↑m + nim ↑m_1) = ↑(m ^^^ m_1) m : ℕ hm : ∀ m_1 < m, grundyValue (nim ↑n + nim ↑m_1) = ↑(n ^^^ m_1) i : LeftMoves (nim ↑n + nim ↑m) a : LeftMoves (nim ↑m) k : ℕ hk : k < m ⊢ grundyValue (nim ↑n + nim ↑k) ≠ ↑(n ^^^ m)
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq]; exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h⟩ #align pgame.grundy_value_eq_iff_equiv_nim SetTheory.PGame.grundyValue_eq_iff_equiv_nim @[simp] theorem nim_grundyValue (o : Ordinal.{u}) : grundyValue (nim o) = o := grundyValue_eq_iff_equiv_nim.2 PGame.equiv_rfl #align pgame.nim_grundy_value SetTheory.PGame.nim_grundyValue theorem grundyValue_eq_iff_equiv (G H : PGame) [G.Impartial] [H.Impartial] : grundyValue G = grundyValue H ↔ (G ≈ H) := grundyValue_eq_iff_equiv_nim.trans (equiv_congr_left.1 (equiv_nim_grundyValue H) _).symm #align pgame.grundy_value_eq_iff_equiv SetTheory.PGame.grundyValue_eq_iff_equiv @[simp] theorem grundyValue_zero : grundyValue 0 = 0 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_zero_equiv) #align pgame.grundy_value_zero SetTheory.PGame.grundyValue_zero theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by rw [← grundyValue_eq_iff_equiv, grundyValue_zero] #align pgame.grundy_value_iff_equiv_zero SetTheory.PGame.grundyValue_iff_equiv_zero @[simp] theorem grundyValue_star : grundyValue star = 1 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_one_equiv) #align pgame.grundy_value_star SetTheory.PGame.grundyValue_star @[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G := by rw [grundyValue_eq_iff_equiv_nim, neg_equiv_iff, neg_nim, ← grundyValue_eq_iff_equiv_nim] #align pgame.grundy_value_neg SetTheory.PGame.grundyValue_neg theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i haveI : (R i).Impartial := @Impartial.moveRight_impartial ⟨l, r, L, R⟩ _ i apply grundyValue_neg #align pgame.grundy_value_eq_mex_right SetTheory.PGame.grundyValue_eq_mex_right -- Todo: this actually generalizes to all ordinals, by defining `Ordinal.lxor` as the pairwise -- `Nat.xor` of base `ω` Cantor normal forms. /-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk
first | rw [hn _ hk] | rw [hm _ hk]
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk
Mathlib.SetTheory.Game.Nim.360_0.mmFMhRYSjViKjcP
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m
Mathlib_SetTheory_Game_Nim
case h.h.refine_1.hr.intro n : ℕ hn : ∀ m < n, ∀ (m_1 : ℕ), grundyValue (nim ↑m + nim ↑m_1) = ↑(m ^^^ m_1) m : ℕ hm : ∀ m_1 < m, grundyValue (nim ↑n + nim ↑m_1) = ↑(n ^^^ m_1) i : LeftMoves (nim ↑n + nim ↑m) a : LeftMoves (nim ↑m) k : ℕ hk : k < m ⊢ grundyValue (nim ↑n + nim ↑k) ≠ ↑(n ^^^ m)
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq]; exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h⟩ #align pgame.grundy_value_eq_iff_equiv_nim SetTheory.PGame.grundyValue_eq_iff_equiv_nim @[simp] theorem nim_grundyValue (o : Ordinal.{u}) : grundyValue (nim o) = o := grundyValue_eq_iff_equiv_nim.2 PGame.equiv_rfl #align pgame.nim_grundy_value SetTheory.PGame.nim_grundyValue theorem grundyValue_eq_iff_equiv (G H : PGame) [G.Impartial] [H.Impartial] : grundyValue G = grundyValue H ↔ (G ≈ H) := grundyValue_eq_iff_equiv_nim.trans (equiv_congr_left.1 (equiv_nim_grundyValue H) _).symm #align pgame.grundy_value_eq_iff_equiv SetTheory.PGame.grundyValue_eq_iff_equiv @[simp] theorem grundyValue_zero : grundyValue 0 = 0 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_zero_equiv) #align pgame.grundy_value_zero SetTheory.PGame.grundyValue_zero theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by rw [← grundyValue_eq_iff_equiv, grundyValue_zero] #align pgame.grundy_value_iff_equiv_zero SetTheory.PGame.grundyValue_iff_equiv_zero @[simp] theorem grundyValue_star : grundyValue star = 1 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_one_equiv) #align pgame.grundy_value_star SetTheory.PGame.grundyValue_star @[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G := by rw [grundyValue_eq_iff_equiv_nim, neg_equiv_iff, neg_nim, ← grundyValue_eq_iff_equiv_nim] #align pgame.grundy_value_neg SetTheory.PGame.grundyValue_neg theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i haveI : (R i).Impartial := @Impartial.moveRight_impartial ⟨l, r, L, R⟩ _ i apply grundyValue_neg #align pgame.grundy_value_eq_mex_right SetTheory.PGame.grundyValue_eq_mex_right -- Todo: this actually generalizes to all ordinals, by defining `Ordinal.lxor` as the pairwise -- `Nat.xor` of base `ω` Cantor normal forms. /-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk first |
rw [hn _ hk]
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk first |
Mathlib.SetTheory.Game.Nim.360_0.mmFMhRYSjViKjcP
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m
Mathlib_SetTheory_Game_Nim
case h.h.refine_1.hr.intro n : ℕ hn : ∀ m < n, ∀ (m_1 : ℕ), grundyValue (nim ↑m + nim ↑m_1) = ↑(m ^^^ m_1) m : ℕ hm : ∀ m_1 < m, grundyValue (nim ↑n + nim ↑m_1) = ↑(n ^^^ m_1) i : LeftMoves (nim ↑n + nim ↑m) a : LeftMoves (nim ↑m) k : ℕ hk : k < m ⊢ grundyValue (nim ↑n + nim ↑k) ≠ ↑(n ^^^ m)
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq]; exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h⟩ #align pgame.grundy_value_eq_iff_equiv_nim SetTheory.PGame.grundyValue_eq_iff_equiv_nim @[simp] theorem nim_grundyValue (o : Ordinal.{u}) : grundyValue (nim o) = o := grundyValue_eq_iff_equiv_nim.2 PGame.equiv_rfl #align pgame.nim_grundy_value SetTheory.PGame.nim_grundyValue theorem grundyValue_eq_iff_equiv (G H : PGame) [G.Impartial] [H.Impartial] : grundyValue G = grundyValue H ↔ (G ≈ H) := grundyValue_eq_iff_equiv_nim.trans (equiv_congr_left.1 (equiv_nim_grundyValue H) _).symm #align pgame.grundy_value_eq_iff_equiv SetTheory.PGame.grundyValue_eq_iff_equiv @[simp] theorem grundyValue_zero : grundyValue 0 = 0 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_zero_equiv) #align pgame.grundy_value_zero SetTheory.PGame.grundyValue_zero theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by rw [← grundyValue_eq_iff_equiv, grundyValue_zero] #align pgame.grundy_value_iff_equiv_zero SetTheory.PGame.grundyValue_iff_equiv_zero @[simp] theorem grundyValue_star : grundyValue star = 1 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_one_equiv) #align pgame.grundy_value_star SetTheory.PGame.grundyValue_star @[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G := by rw [grundyValue_eq_iff_equiv_nim, neg_equiv_iff, neg_nim, ← grundyValue_eq_iff_equiv_nim] #align pgame.grundy_value_neg SetTheory.PGame.grundyValue_neg theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i haveI : (R i).Impartial := @Impartial.moveRight_impartial ⟨l, r, L, R⟩ _ i apply grundyValue_neg #align pgame.grundy_value_eq_mex_right SetTheory.PGame.grundyValue_eq_mex_right -- Todo: this actually generalizes to all ordinals, by defining `Ordinal.lxor` as the pairwise -- `Nat.xor` of base `ω` Cantor normal forms. /-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk first | rw [hn _ hk] |
rw [hm _ hk]
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk first | rw [hn _ hk] |
Mathlib.SetTheory.Game.Nim.360_0.mmFMhRYSjViKjcP
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m
Mathlib_SetTheory_Game_Nim
case h.h.refine_1.hr.intro n : ℕ hn : ∀ m < n, ∀ (m_1 : ℕ), grundyValue (nim ↑m + nim ↑m_1) = ↑(m ^^^ m_1) m : ℕ hm : ∀ m_1 < m, grundyValue (nim ↑n + nim ↑m_1) = ↑(n ^^^ m_1) i : LeftMoves (nim ↑n + nim ↑m) a : LeftMoves (nim ↑m) k : ℕ hk : k < m ⊢ ↑(n ^^^ k) ≠ ↑(n ^^^ m)
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq]; exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h⟩ #align pgame.grundy_value_eq_iff_equiv_nim SetTheory.PGame.grundyValue_eq_iff_equiv_nim @[simp] theorem nim_grundyValue (o : Ordinal.{u}) : grundyValue (nim o) = o := grundyValue_eq_iff_equiv_nim.2 PGame.equiv_rfl #align pgame.nim_grundy_value SetTheory.PGame.nim_grundyValue theorem grundyValue_eq_iff_equiv (G H : PGame) [G.Impartial] [H.Impartial] : grundyValue G = grundyValue H ↔ (G ≈ H) := grundyValue_eq_iff_equiv_nim.trans (equiv_congr_left.1 (equiv_nim_grundyValue H) _).symm #align pgame.grundy_value_eq_iff_equiv SetTheory.PGame.grundyValue_eq_iff_equiv @[simp] theorem grundyValue_zero : grundyValue 0 = 0 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_zero_equiv) #align pgame.grundy_value_zero SetTheory.PGame.grundyValue_zero theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by rw [← grundyValue_eq_iff_equiv, grundyValue_zero] #align pgame.grundy_value_iff_equiv_zero SetTheory.PGame.grundyValue_iff_equiv_zero @[simp] theorem grundyValue_star : grundyValue star = 1 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_one_equiv) #align pgame.grundy_value_star SetTheory.PGame.grundyValue_star @[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G := by rw [grundyValue_eq_iff_equiv_nim, neg_equiv_iff, neg_nim, ← grundyValue_eq_iff_equiv_nim] #align pgame.grundy_value_neg SetTheory.PGame.grundyValue_neg theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i haveI : (R i).Impartial := @Impartial.moveRight_impartial ⟨l, r, L, R⟩ _ i apply grundyValue_neg #align pgame.grundy_value_eq_mex_right SetTheory.PGame.grundyValue_eq_mex_right -- Todo: this actually generalizes to all ordinals, by defining `Ordinal.lxor` as the pairwise -- `Nat.xor` of base `ω` Cantor normal forms. /-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk first | rw [hn _ hk] | rw [hm _ hk]
refine' fun h => hk.ne _
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk first | rw [hn _ hk] | rw [hm _ hk]
Mathlib.SetTheory.Game.Nim.360_0.mmFMhRYSjViKjcP
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m
Mathlib_SetTheory_Game_Nim
case h.h.refine_1.hr.intro n : ℕ hn : ∀ m < n, ∀ (m_1 : ℕ), grundyValue (nim ↑m + nim ↑m_1) = ↑(m ^^^ m_1) m : ℕ hm : ∀ m_1 < m, grundyValue (nim ↑n + nim ↑m_1) = ↑(n ^^^ m_1) i : LeftMoves (nim ↑n + nim ↑m) a : LeftMoves (nim ↑m) k : ℕ hk : k < m h : ↑(n ^^^ k) = ↑(n ^^^ m) ⊢ k = m
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq]; exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h⟩ #align pgame.grundy_value_eq_iff_equiv_nim SetTheory.PGame.grundyValue_eq_iff_equiv_nim @[simp] theorem nim_grundyValue (o : Ordinal.{u}) : grundyValue (nim o) = o := grundyValue_eq_iff_equiv_nim.2 PGame.equiv_rfl #align pgame.nim_grundy_value SetTheory.PGame.nim_grundyValue theorem grundyValue_eq_iff_equiv (G H : PGame) [G.Impartial] [H.Impartial] : grundyValue G = grundyValue H ↔ (G ≈ H) := grundyValue_eq_iff_equiv_nim.trans (equiv_congr_left.1 (equiv_nim_grundyValue H) _).symm #align pgame.grundy_value_eq_iff_equiv SetTheory.PGame.grundyValue_eq_iff_equiv @[simp] theorem grundyValue_zero : grundyValue 0 = 0 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_zero_equiv) #align pgame.grundy_value_zero SetTheory.PGame.grundyValue_zero theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by rw [← grundyValue_eq_iff_equiv, grundyValue_zero] #align pgame.grundy_value_iff_equiv_zero SetTheory.PGame.grundyValue_iff_equiv_zero @[simp] theorem grundyValue_star : grundyValue star = 1 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_one_equiv) #align pgame.grundy_value_star SetTheory.PGame.grundyValue_star @[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G := by rw [grundyValue_eq_iff_equiv_nim, neg_equiv_iff, neg_nim, ← grundyValue_eq_iff_equiv_nim] #align pgame.grundy_value_neg SetTheory.PGame.grundyValue_neg theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i haveI : (R i).Impartial := @Impartial.moveRight_impartial ⟨l, r, L, R⟩ _ i apply grundyValue_neg #align pgame.grundy_value_eq_mex_right SetTheory.PGame.grundyValue_eq_mex_right -- Todo: this actually generalizes to all ordinals, by defining `Ordinal.lxor` as the pairwise -- `Nat.xor` of base `ω` Cantor normal forms. /-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk first | rw [hn _ hk] | rw [hm _ hk] refine' fun h => hk.ne _
rw [Ordinal.nat_cast_inj] at h
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk first | rw [hn _ hk] | rw [hm _ hk] refine' fun h => hk.ne _
Mathlib.SetTheory.Game.Nim.360_0.mmFMhRYSjViKjcP
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m
Mathlib_SetTheory_Game_Nim
case h.h.refine_1.hr.intro n : ℕ hn : ∀ m < n, ∀ (m_1 : ℕ), grundyValue (nim ↑m + nim ↑m_1) = ↑(m ^^^ m_1) m : ℕ hm : ∀ m_1 < m, grundyValue (nim ↑n + nim ↑m_1) = ↑(n ^^^ m_1) i : LeftMoves (nim ↑n + nim ↑m) a : LeftMoves (nim ↑m) k : ℕ hk : k < m h : n ^^^ k = n ^^^ m ⊢ k = m
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq]; exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h⟩ #align pgame.grundy_value_eq_iff_equiv_nim SetTheory.PGame.grundyValue_eq_iff_equiv_nim @[simp] theorem nim_grundyValue (o : Ordinal.{u}) : grundyValue (nim o) = o := grundyValue_eq_iff_equiv_nim.2 PGame.equiv_rfl #align pgame.nim_grundy_value SetTheory.PGame.nim_grundyValue theorem grundyValue_eq_iff_equiv (G H : PGame) [G.Impartial] [H.Impartial] : grundyValue G = grundyValue H ↔ (G ≈ H) := grundyValue_eq_iff_equiv_nim.trans (equiv_congr_left.1 (equiv_nim_grundyValue H) _).symm #align pgame.grundy_value_eq_iff_equiv SetTheory.PGame.grundyValue_eq_iff_equiv @[simp] theorem grundyValue_zero : grundyValue 0 = 0 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_zero_equiv) #align pgame.grundy_value_zero SetTheory.PGame.grundyValue_zero theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by rw [← grundyValue_eq_iff_equiv, grundyValue_zero] #align pgame.grundy_value_iff_equiv_zero SetTheory.PGame.grundyValue_iff_equiv_zero @[simp] theorem grundyValue_star : grundyValue star = 1 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_one_equiv) #align pgame.grundy_value_star SetTheory.PGame.grundyValue_star @[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G := by rw [grundyValue_eq_iff_equiv_nim, neg_equiv_iff, neg_nim, ← grundyValue_eq_iff_equiv_nim] #align pgame.grundy_value_neg SetTheory.PGame.grundyValue_neg theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i haveI : (R i).Impartial := @Impartial.moveRight_impartial ⟨l, r, L, R⟩ _ i apply grundyValue_neg #align pgame.grundy_value_eq_mex_right SetTheory.PGame.grundyValue_eq_mex_right -- Todo: this actually generalizes to all ordinals, by defining `Ordinal.lxor` as the pairwise -- `Nat.xor` of base `ω` Cantor normal forms. /-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk first | rw [hn _ hk] | rw [hm _ hk] refine' fun h => hk.ne _ rw [Ordinal.nat_cast_inj] at h
first | rwa [Nat.xor_left_inj] at h | rwa [Nat.xor_right_inj] at h
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk first | rw [hn _ hk] | rw [hm _ hk] refine' fun h => hk.ne _ rw [Ordinal.nat_cast_inj] at h
Mathlib.SetTheory.Game.Nim.360_0.mmFMhRYSjViKjcP
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m
Mathlib_SetTheory_Game_Nim
case h.h.refine_1.hr.intro n : ℕ hn : ∀ m < n, ∀ (m_1 : ℕ), grundyValue (nim ↑m + nim ↑m_1) = ↑(m ^^^ m_1) m : ℕ hm : ∀ m_1 < m, grundyValue (nim ↑n + nim ↑m_1) = ↑(n ^^^ m_1) i : LeftMoves (nim ↑n + nim ↑m) a : LeftMoves (nim ↑m) k : ℕ hk : k < m h : n ^^^ k = n ^^^ m ⊢ k = m
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq]; exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h⟩ #align pgame.grundy_value_eq_iff_equiv_nim SetTheory.PGame.grundyValue_eq_iff_equiv_nim @[simp] theorem nim_grundyValue (o : Ordinal.{u}) : grundyValue (nim o) = o := grundyValue_eq_iff_equiv_nim.2 PGame.equiv_rfl #align pgame.nim_grundy_value SetTheory.PGame.nim_grundyValue theorem grundyValue_eq_iff_equiv (G H : PGame) [G.Impartial] [H.Impartial] : grundyValue G = grundyValue H ↔ (G ≈ H) := grundyValue_eq_iff_equiv_nim.trans (equiv_congr_left.1 (equiv_nim_grundyValue H) _).symm #align pgame.grundy_value_eq_iff_equiv SetTheory.PGame.grundyValue_eq_iff_equiv @[simp] theorem grundyValue_zero : grundyValue 0 = 0 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_zero_equiv) #align pgame.grundy_value_zero SetTheory.PGame.grundyValue_zero theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by rw [← grundyValue_eq_iff_equiv, grundyValue_zero] #align pgame.grundy_value_iff_equiv_zero SetTheory.PGame.grundyValue_iff_equiv_zero @[simp] theorem grundyValue_star : grundyValue star = 1 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_one_equiv) #align pgame.grundy_value_star SetTheory.PGame.grundyValue_star @[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G := by rw [grundyValue_eq_iff_equiv_nim, neg_equiv_iff, neg_nim, ← grundyValue_eq_iff_equiv_nim] #align pgame.grundy_value_neg SetTheory.PGame.grundyValue_neg theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i haveI : (R i).Impartial := @Impartial.moveRight_impartial ⟨l, r, L, R⟩ _ i apply grundyValue_neg #align pgame.grundy_value_eq_mex_right SetTheory.PGame.grundyValue_eq_mex_right -- Todo: this actually generalizes to all ordinals, by defining `Ordinal.lxor` as the pairwise -- `Nat.xor` of base `ω` Cantor normal forms. /-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk first | rw [hn _ hk] | rw [hm _ hk] refine' fun h => hk.ne _ rw [Ordinal.nat_cast_inj] at h first |
rwa [Nat.xor_left_inj] at h
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk first | rw [hn _ hk] | rw [hm _ hk] refine' fun h => hk.ne _ rw [Ordinal.nat_cast_inj] at h first |
Mathlib.SetTheory.Game.Nim.360_0.mmFMhRYSjViKjcP
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m
Mathlib_SetTheory_Game_Nim
case h.h.refine_1.hr.intro n : ℕ hn : ∀ m < n, ∀ (m_1 : ℕ), grundyValue (nim ↑m + nim ↑m_1) = ↑(m ^^^ m_1) m : ℕ hm : ∀ m_1 < m, grundyValue (nim ↑n + nim ↑m_1) = ↑(n ^^^ m_1) i : LeftMoves (nim ↑n + nim ↑m) a : LeftMoves (nim ↑m) k : ℕ hk : k < m h : n ^^^ k = n ^^^ m ⊢ k = m
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq]; exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h⟩ #align pgame.grundy_value_eq_iff_equiv_nim SetTheory.PGame.grundyValue_eq_iff_equiv_nim @[simp] theorem nim_grundyValue (o : Ordinal.{u}) : grundyValue (nim o) = o := grundyValue_eq_iff_equiv_nim.2 PGame.equiv_rfl #align pgame.nim_grundy_value SetTheory.PGame.nim_grundyValue theorem grundyValue_eq_iff_equiv (G H : PGame) [G.Impartial] [H.Impartial] : grundyValue G = grundyValue H ↔ (G ≈ H) := grundyValue_eq_iff_equiv_nim.trans (equiv_congr_left.1 (equiv_nim_grundyValue H) _).symm #align pgame.grundy_value_eq_iff_equiv SetTheory.PGame.grundyValue_eq_iff_equiv @[simp] theorem grundyValue_zero : grundyValue 0 = 0 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_zero_equiv) #align pgame.grundy_value_zero SetTheory.PGame.grundyValue_zero theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by rw [← grundyValue_eq_iff_equiv, grundyValue_zero] #align pgame.grundy_value_iff_equiv_zero SetTheory.PGame.grundyValue_iff_equiv_zero @[simp] theorem grundyValue_star : grundyValue star = 1 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_one_equiv) #align pgame.grundy_value_star SetTheory.PGame.grundyValue_star @[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G := by rw [grundyValue_eq_iff_equiv_nim, neg_equiv_iff, neg_nim, ← grundyValue_eq_iff_equiv_nim] #align pgame.grundy_value_neg SetTheory.PGame.grundyValue_neg theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i haveI : (R i).Impartial := @Impartial.moveRight_impartial ⟨l, r, L, R⟩ _ i apply grundyValue_neg #align pgame.grundy_value_eq_mex_right SetTheory.PGame.grundyValue_eq_mex_right -- Todo: this actually generalizes to all ordinals, by defining `Ordinal.lxor` as the pairwise -- `Nat.xor` of base `ω` Cantor normal forms. /-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk first | rw [hn _ hk] | rw [hm _ hk] refine' fun h => hk.ne _ rw [Ordinal.nat_cast_inj] at h first | rwa [Nat.xor_left_inj] at h |
rwa [Nat.xor_right_inj] at h
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk first | rw [hn _ hk] | rw [hm _ hk] refine' fun h => hk.ne _ rw [Ordinal.nat_cast_inj] at h first | rwa [Nat.xor_left_inj] at h |
Mathlib.SetTheory.Game.Nim.360_0.mmFMhRYSjViKjcP
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m
Mathlib_SetTheory_Game_Nim
case h.h.refine_2 n : ℕ hn : ∀ m < n, ∀ (m_1 : ℕ), grundyValue (nim ↑m + nim ↑m_1) = ↑(m ^^^ m_1) m : ℕ hm : ∀ m_1 < m, grundyValue (nim ↑n + nim ↑m_1) = ↑(n ^^^ m_1) ou : Ordinal.{u} hu : ou < ↑(n ^^^ m) ⊢ ∃ i, grundyValue (moveLeft (nim ↑n + nim ↑m) i) = ou
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq]; exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h⟩ #align pgame.grundy_value_eq_iff_equiv_nim SetTheory.PGame.grundyValue_eq_iff_equiv_nim @[simp] theorem nim_grundyValue (o : Ordinal.{u}) : grundyValue (nim o) = o := grundyValue_eq_iff_equiv_nim.2 PGame.equiv_rfl #align pgame.nim_grundy_value SetTheory.PGame.nim_grundyValue theorem grundyValue_eq_iff_equiv (G H : PGame) [G.Impartial] [H.Impartial] : grundyValue G = grundyValue H ↔ (G ≈ H) := grundyValue_eq_iff_equiv_nim.trans (equiv_congr_left.1 (equiv_nim_grundyValue H) _).symm #align pgame.grundy_value_eq_iff_equiv SetTheory.PGame.grundyValue_eq_iff_equiv @[simp] theorem grundyValue_zero : grundyValue 0 = 0 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_zero_equiv) #align pgame.grundy_value_zero SetTheory.PGame.grundyValue_zero theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by rw [← grundyValue_eq_iff_equiv, grundyValue_zero] #align pgame.grundy_value_iff_equiv_zero SetTheory.PGame.grundyValue_iff_equiv_zero @[simp] theorem grundyValue_star : grundyValue star = 1 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_one_equiv) #align pgame.grundy_value_star SetTheory.PGame.grundyValue_star @[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G := by rw [grundyValue_eq_iff_equiv_nim, neg_equiv_iff, neg_nim, ← grundyValue_eq_iff_equiv_nim] #align pgame.grundy_value_neg SetTheory.PGame.grundyValue_neg theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i haveI : (R i).Impartial := @Impartial.moveRight_impartial ⟨l, r, L, R⟩ _ i apply grundyValue_neg #align pgame.grundy_value_eq_mex_right SetTheory.PGame.grundyValue_eq_mex_right -- Todo: this actually generalizes to all ordinals, by defining `Ordinal.lxor` as the pairwise -- `Nat.xor` of base `ω` Cantor normal forms. /-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk first | rw [hn _ hk] | rw [hm _ hk] refine' fun h => hk.ne _ rw [Ordinal.nat_cast_inj] at h first | rwa [Nat.xor_left_inj] at h | rwa [Nat.xor_right_inj] at h -- Every other smaller Grundy value can be reached by left moves. · -- If `u < m ^^^ n`, then either `u ^^^ n < m` or `u ^^^ m < n`.
obtain ⟨u, rfl⟩ := Ordinal.lt_omega.1 (hu.trans (Ordinal.nat_lt_omega _))
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk first | rw [hn _ hk] | rw [hm _ hk] refine' fun h => hk.ne _ rw [Ordinal.nat_cast_inj] at h first | rwa [Nat.xor_left_inj] at h | rwa [Nat.xor_right_inj] at h -- Every other smaller Grundy value can be reached by left moves. · -- If `u < m ^^^ n`, then either `u ^^^ n < m` or `u ^^^ m < n`.
Mathlib.SetTheory.Game.Nim.360_0.mmFMhRYSjViKjcP
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m
Mathlib_SetTheory_Game_Nim
case h.h.refine_2.intro n : ℕ hn : ∀ m < n, ∀ (m_1 : ℕ), grundyValue (nim ↑m + nim ↑m_1) = ↑(m ^^^ m_1) m : ℕ hm : ∀ m_1 < m, grundyValue (nim ↑n + nim ↑m_1) = ↑(n ^^^ m_1) u : ℕ hu : ↑u < ↑(n ^^^ m) ⊢ ∃ i, grundyValue (moveLeft (nim ↑n + nim ↑m) i) = ↑u
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq]; exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h⟩ #align pgame.grundy_value_eq_iff_equiv_nim SetTheory.PGame.grundyValue_eq_iff_equiv_nim @[simp] theorem nim_grundyValue (o : Ordinal.{u}) : grundyValue (nim o) = o := grundyValue_eq_iff_equiv_nim.2 PGame.equiv_rfl #align pgame.nim_grundy_value SetTheory.PGame.nim_grundyValue theorem grundyValue_eq_iff_equiv (G H : PGame) [G.Impartial] [H.Impartial] : grundyValue G = grundyValue H ↔ (G ≈ H) := grundyValue_eq_iff_equiv_nim.trans (equiv_congr_left.1 (equiv_nim_grundyValue H) _).symm #align pgame.grundy_value_eq_iff_equiv SetTheory.PGame.grundyValue_eq_iff_equiv @[simp] theorem grundyValue_zero : grundyValue 0 = 0 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_zero_equiv) #align pgame.grundy_value_zero SetTheory.PGame.grundyValue_zero theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by rw [← grundyValue_eq_iff_equiv, grundyValue_zero] #align pgame.grundy_value_iff_equiv_zero SetTheory.PGame.grundyValue_iff_equiv_zero @[simp] theorem grundyValue_star : grundyValue star = 1 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_one_equiv) #align pgame.grundy_value_star SetTheory.PGame.grundyValue_star @[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G := by rw [grundyValue_eq_iff_equiv_nim, neg_equiv_iff, neg_nim, ← grundyValue_eq_iff_equiv_nim] #align pgame.grundy_value_neg SetTheory.PGame.grundyValue_neg theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i haveI : (R i).Impartial := @Impartial.moveRight_impartial ⟨l, r, L, R⟩ _ i apply grundyValue_neg #align pgame.grundy_value_eq_mex_right SetTheory.PGame.grundyValue_eq_mex_right -- Todo: this actually generalizes to all ordinals, by defining `Ordinal.lxor` as the pairwise -- `Nat.xor` of base `ω` Cantor normal forms. /-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk first | rw [hn _ hk] | rw [hm _ hk] refine' fun h => hk.ne _ rw [Ordinal.nat_cast_inj] at h first | rwa [Nat.xor_left_inj] at h | rwa [Nat.xor_right_inj] at h -- Every other smaller Grundy value can be reached by left moves. · -- If `u < m ^^^ n`, then either `u ^^^ n < m` or `u ^^^ m < n`. obtain ⟨u, rfl⟩ := Ordinal.lt_omega.1 (hu.trans (Ordinal.nat_lt_omega _))
replace hu := Ordinal.nat_cast_lt.1 hu
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk first | rw [hn _ hk] | rw [hm _ hk] refine' fun h => hk.ne _ rw [Ordinal.nat_cast_inj] at h first | rwa [Nat.xor_left_inj] at h | rwa [Nat.xor_right_inj] at h -- Every other smaller Grundy value can be reached by left moves. · -- If `u < m ^^^ n`, then either `u ^^^ n < m` or `u ^^^ m < n`. obtain ⟨u, rfl⟩ := Ordinal.lt_omega.1 (hu.trans (Ordinal.nat_lt_omega _))
Mathlib.SetTheory.Game.Nim.360_0.mmFMhRYSjViKjcP
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m
Mathlib_SetTheory_Game_Nim
case h.h.refine_2.intro n : ℕ hn : ∀ m < n, ∀ (m_1 : ℕ), grundyValue (nim ↑m + nim ↑m_1) = ↑(m ^^^ m_1) m : ℕ hm : ∀ m_1 < m, grundyValue (nim ↑n + nim ↑m_1) = ↑(n ^^^ m_1) u : ℕ hu : u < n ^^^ m ⊢ ∃ i, grundyValue (moveLeft (nim ↑n + nim ↑m) i) = ↑u
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq]; exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h⟩ #align pgame.grundy_value_eq_iff_equiv_nim SetTheory.PGame.grundyValue_eq_iff_equiv_nim @[simp] theorem nim_grundyValue (o : Ordinal.{u}) : grundyValue (nim o) = o := grundyValue_eq_iff_equiv_nim.2 PGame.equiv_rfl #align pgame.nim_grundy_value SetTheory.PGame.nim_grundyValue theorem grundyValue_eq_iff_equiv (G H : PGame) [G.Impartial] [H.Impartial] : grundyValue G = grundyValue H ↔ (G ≈ H) := grundyValue_eq_iff_equiv_nim.trans (equiv_congr_left.1 (equiv_nim_grundyValue H) _).symm #align pgame.grundy_value_eq_iff_equiv SetTheory.PGame.grundyValue_eq_iff_equiv @[simp] theorem grundyValue_zero : grundyValue 0 = 0 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_zero_equiv) #align pgame.grundy_value_zero SetTheory.PGame.grundyValue_zero theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by rw [← grundyValue_eq_iff_equiv, grundyValue_zero] #align pgame.grundy_value_iff_equiv_zero SetTheory.PGame.grundyValue_iff_equiv_zero @[simp] theorem grundyValue_star : grundyValue star = 1 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_one_equiv) #align pgame.grundy_value_star SetTheory.PGame.grundyValue_star @[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G := by rw [grundyValue_eq_iff_equiv_nim, neg_equiv_iff, neg_nim, ← grundyValue_eq_iff_equiv_nim] #align pgame.grundy_value_neg SetTheory.PGame.grundyValue_neg theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i haveI : (R i).Impartial := @Impartial.moveRight_impartial ⟨l, r, L, R⟩ _ i apply grundyValue_neg #align pgame.grundy_value_eq_mex_right SetTheory.PGame.grundyValue_eq_mex_right -- Todo: this actually generalizes to all ordinals, by defining `Ordinal.lxor` as the pairwise -- `Nat.xor` of base `ω` Cantor normal forms. /-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk first | rw [hn _ hk] | rw [hm _ hk] refine' fun h => hk.ne _ rw [Ordinal.nat_cast_inj] at h first | rwa [Nat.xor_left_inj] at h | rwa [Nat.xor_right_inj] at h -- Every other smaller Grundy value can be reached by left moves. · -- If `u < m ^^^ n`, then either `u ^^^ n < m` or `u ^^^ m < n`. obtain ⟨u, rfl⟩ := Ordinal.lt_omega.1 (hu.trans (Ordinal.nat_lt_omega _)) replace hu := Ordinal.nat_cast_lt.1 hu
cases' Nat.lt_xor_cases hu with h h
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk first | rw [hn _ hk] | rw [hm _ hk] refine' fun h => hk.ne _ rw [Ordinal.nat_cast_inj] at h first | rwa [Nat.xor_left_inj] at h | rwa [Nat.xor_right_inj] at h -- Every other smaller Grundy value can be reached by left moves. · -- If `u < m ^^^ n`, then either `u ^^^ n < m` or `u ^^^ m < n`. obtain ⟨u, rfl⟩ := Ordinal.lt_omega.1 (hu.trans (Ordinal.nat_lt_omega _)) replace hu := Ordinal.nat_cast_lt.1 hu
Mathlib.SetTheory.Game.Nim.360_0.mmFMhRYSjViKjcP
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m
Mathlib_SetTheory_Game_Nim
case h.h.refine_2.intro.inl n : ℕ hn : ∀ m < n, ∀ (m_1 : ℕ), grundyValue (nim ↑m + nim ↑m_1) = ↑(m ^^^ m_1) m : ℕ hm : ∀ m_1 < m, grundyValue (nim ↑n + nim ↑m_1) = ↑(n ^^^ m_1) u : ℕ hu : u < n ^^^ m h : u ^^^ m < n ⊢ ∃ i, grundyValue (moveLeft (nim ↑n + nim ↑m) i) = ↑u
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq]; exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h⟩ #align pgame.grundy_value_eq_iff_equiv_nim SetTheory.PGame.grundyValue_eq_iff_equiv_nim @[simp] theorem nim_grundyValue (o : Ordinal.{u}) : grundyValue (nim o) = o := grundyValue_eq_iff_equiv_nim.2 PGame.equiv_rfl #align pgame.nim_grundy_value SetTheory.PGame.nim_grundyValue theorem grundyValue_eq_iff_equiv (G H : PGame) [G.Impartial] [H.Impartial] : grundyValue G = grundyValue H ↔ (G ≈ H) := grundyValue_eq_iff_equiv_nim.trans (equiv_congr_left.1 (equiv_nim_grundyValue H) _).symm #align pgame.grundy_value_eq_iff_equiv SetTheory.PGame.grundyValue_eq_iff_equiv @[simp] theorem grundyValue_zero : grundyValue 0 = 0 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_zero_equiv) #align pgame.grundy_value_zero SetTheory.PGame.grundyValue_zero theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by rw [← grundyValue_eq_iff_equiv, grundyValue_zero] #align pgame.grundy_value_iff_equiv_zero SetTheory.PGame.grundyValue_iff_equiv_zero @[simp] theorem grundyValue_star : grundyValue star = 1 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_one_equiv) #align pgame.grundy_value_star SetTheory.PGame.grundyValue_star @[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G := by rw [grundyValue_eq_iff_equiv_nim, neg_equiv_iff, neg_nim, ← grundyValue_eq_iff_equiv_nim] #align pgame.grundy_value_neg SetTheory.PGame.grundyValue_neg theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i haveI : (R i).Impartial := @Impartial.moveRight_impartial ⟨l, r, L, R⟩ _ i apply grundyValue_neg #align pgame.grundy_value_eq_mex_right SetTheory.PGame.grundyValue_eq_mex_right -- Todo: this actually generalizes to all ordinals, by defining `Ordinal.lxor` as the pairwise -- `Nat.xor` of base `ω` Cantor normal forms. /-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk first | rw [hn _ hk] | rw [hm _ hk] refine' fun h => hk.ne _ rw [Ordinal.nat_cast_inj] at h first | rwa [Nat.xor_left_inj] at h | rwa [Nat.xor_right_inj] at h -- Every other smaller Grundy value can be reached by left moves. · -- If `u < m ^^^ n`, then either `u ^^^ n < m` or `u ^^^ m < n`. obtain ⟨u, rfl⟩ := Ordinal.lt_omega.1 (hu.trans (Ordinal.nat_lt_omega _)) replace hu := Ordinal.nat_cast_lt.1 hu cases' Nat.lt_xor_cases hu with h h -- In the first case, reducing the `m` pile to `u ^^^ n` gives the desired Grundy value. ·
refine' ⟨toLeftMovesAdd (Sum.inl <| toLeftMovesNim ⟨_, Ordinal.nat_cast_lt.2 h⟩), _⟩
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk first | rw [hn _ hk] | rw [hm _ hk] refine' fun h => hk.ne _ rw [Ordinal.nat_cast_inj] at h first | rwa [Nat.xor_left_inj] at h | rwa [Nat.xor_right_inj] at h -- Every other smaller Grundy value can be reached by left moves. · -- If `u < m ^^^ n`, then either `u ^^^ n < m` or `u ^^^ m < n`. obtain ⟨u, rfl⟩ := Ordinal.lt_omega.1 (hu.trans (Ordinal.nat_lt_omega _)) replace hu := Ordinal.nat_cast_lt.1 hu cases' Nat.lt_xor_cases hu with h h -- In the first case, reducing the `m` pile to `u ^^^ n` gives the desired Grundy value. ·
Mathlib.SetTheory.Game.Nim.360_0.mmFMhRYSjViKjcP
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m
Mathlib_SetTheory_Game_Nim
case h.h.refine_2.intro.inl n : ℕ hn : ∀ m < n, ∀ (m_1 : ℕ), grundyValue (nim ↑m + nim ↑m_1) = ↑(m ^^^ m_1) m : ℕ hm : ∀ m_1 < m, grundyValue (nim ↑n + nim ↑m_1) = ↑(n ^^^ m_1) u : ℕ hu : u < n ^^^ m h : u ^^^ m < n ⊢ grundyValue (moveLeft (nim ↑n + nim ↑m) (toLeftMovesAdd (Sum.inl (toLeftMovesNim { val := ↑(u ^^^ m), property := (_ : ↑(u ^^^ m) < ↑n) })))) = ↑u
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq]; exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h⟩ #align pgame.grundy_value_eq_iff_equiv_nim SetTheory.PGame.grundyValue_eq_iff_equiv_nim @[simp] theorem nim_grundyValue (o : Ordinal.{u}) : grundyValue (nim o) = o := grundyValue_eq_iff_equiv_nim.2 PGame.equiv_rfl #align pgame.nim_grundy_value SetTheory.PGame.nim_grundyValue theorem grundyValue_eq_iff_equiv (G H : PGame) [G.Impartial] [H.Impartial] : grundyValue G = grundyValue H ↔ (G ≈ H) := grundyValue_eq_iff_equiv_nim.trans (equiv_congr_left.1 (equiv_nim_grundyValue H) _).symm #align pgame.grundy_value_eq_iff_equiv SetTheory.PGame.grundyValue_eq_iff_equiv @[simp] theorem grundyValue_zero : grundyValue 0 = 0 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_zero_equiv) #align pgame.grundy_value_zero SetTheory.PGame.grundyValue_zero theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by rw [← grundyValue_eq_iff_equiv, grundyValue_zero] #align pgame.grundy_value_iff_equiv_zero SetTheory.PGame.grundyValue_iff_equiv_zero @[simp] theorem grundyValue_star : grundyValue star = 1 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_one_equiv) #align pgame.grundy_value_star SetTheory.PGame.grundyValue_star @[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G := by rw [grundyValue_eq_iff_equiv_nim, neg_equiv_iff, neg_nim, ← grundyValue_eq_iff_equiv_nim] #align pgame.grundy_value_neg SetTheory.PGame.grundyValue_neg theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i haveI : (R i).Impartial := @Impartial.moveRight_impartial ⟨l, r, L, R⟩ _ i apply grundyValue_neg #align pgame.grundy_value_eq_mex_right SetTheory.PGame.grundyValue_eq_mex_right -- Todo: this actually generalizes to all ordinals, by defining `Ordinal.lxor` as the pairwise -- `Nat.xor` of base `ω` Cantor normal forms. /-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk first | rw [hn _ hk] | rw [hm _ hk] refine' fun h => hk.ne _ rw [Ordinal.nat_cast_inj] at h first | rwa [Nat.xor_left_inj] at h | rwa [Nat.xor_right_inj] at h -- Every other smaller Grundy value can be reached by left moves. · -- If `u < m ^^^ n`, then either `u ^^^ n < m` or `u ^^^ m < n`. obtain ⟨u, rfl⟩ := Ordinal.lt_omega.1 (hu.trans (Ordinal.nat_lt_omega _)) replace hu := Ordinal.nat_cast_lt.1 hu cases' Nat.lt_xor_cases hu with h h -- In the first case, reducing the `m` pile to `u ^^^ n` gives the desired Grundy value. · refine' ⟨toLeftMovesAdd (Sum.inl <| toLeftMovesNim ⟨_, Ordinal.nat_cast_lt.2 h⟩), _⟩
simp [Nat.lxor_cancel_right, hn _ h]
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk first | rw [hn _ hk] | rw [hm _ hk] refine' fun h => hk.ne _ rw [Ordinal.nat_cast_inj] at h first | rwa [Nat.xor_left_inj] at h | rwa [Nat.xor_right_inj] at h -- Every other smaller Grundy value can be reached by left moves. · -- If `u < m ^^^ n`, then either `u ^^^ n < m` or `u ^^^ m < n`. obtain ⟨u, rfl⟩ := Ordinal.lt_omega.1 (hu.trans (Ordinal.nat_lt_omega _)) replace hu := Ordinal.nat_cast_lt.1 hu cases' Nat.lt_xor_cases hu with h h -- In the first case, reducing the `m` pile to `u ^^^ n` gives the desired Grundy value. · refine' ⟨toLeftMovesAdd (Sum.inl <| toLeftMovesNim ⟨_, Ordinal.nat_cast_lt.2 h⟩), _⟩
Mathlib.SetTheory.Game.Nim.360_0.mmFMhRYSjViKjcP
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m
Mathlib_SetTheory_Game_Nim
case h.h.refine_2.intro.inr n : ℕ hn : ∀ m < n, ∀ (m_1 : ℕ), grundyValue (nim ↑m + nim ↑m_1) = ↑(m ^^^ m_1) m : ℕ hm : ∀ m_1 < m, grundyValue (nim ↑n + nim ↑m_1) = ↑(n ^^^ m_1) u : ℕ hu : u < n ^^^ m h : u ^^^ n < m ⊢ ∃ i, grundyValue (moveLeft (nim ↑n + nim ↑m) i) = ↑u
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq]; exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h⟩ #align pgame.grundy_value_eq_iff_equiv_nim SetTheory.PGame.grundyValue_eq_iff_equiv_nim @[simp] theorem nim_grundyValue (o : Ordinal.{u}) : grundyValue (nim o) = o := grundyValue_eq_iff_equiv_nim.2 PGame.equiv_rfl #align pgame.nim_grundy_value SetTheory.PGame.nim_grundyValue theorem grundyValue_eq_iff_equiv (G H : PGame) [G.Impartial] [H.Impartial] : grundyValue G = grundyValue H ↔ (G ≈ H) := grundyValue_eq_iff_equiv_nim.trans (equiv_congr_left.1 (equiv_nim_grundyValue H) _).symm #align pgame.grundy_value_eq_iff_equiv SetTheory.PGame.grundyValue_eq_iff_equiv @[simp] theorem grundyValue_zero : grundyValue 0 = 0 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_zero_equiv) #align pgame.grundy_value_zero SetTheory.PGame.grundyValue_zero theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by rw [← grundyValue_eq_iff_equiv, grundyValue_zero] #align pgame.grundy_value_iff_equiv_zero SetTheory.PGame.grundyValue_iff_equiv_zero @[simp] theorem grundyValue_star : grundyValue star = 1 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_one_equiv) #align pgame.grundy_value_star SetTheory.PGame.grundyValue_star @[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G := by rw [grundyValue_eq_iff_equiv_nim, neg_equiv_iff, neg_nim, ← grundyValue_eq_iff_equiv_nim] #align pgame.grundy_value_neg SetTheory.PGame.grundyValue_neg theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i haveI : (R i).Impartial := @Impartial.moveRight_impartial ⟨l, r, L, R⟩ _ i apply grundyValue_neg #align pgame.grundy_value_eq_mex_right SetTheory.PGame.grundyValue_eq_mex_right -- Todo: this actually generalizes to all ordinals, by defining `Ordinal.lxor` as the pairwise -- `Nat.xor` of base `ω` Cantor normal forms. /-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk first | rw [hn _ hk] | rw [hm _ hk] refine' fun h => hk.ne _ rw [Ordinal.nat_cast_inj] at h first | rwa [Nat.xor_left_inj] at h | rwa [Nat.xor_right_inj] at h -- Every other smaller Grundy value can be reached by left moves. · -- If `u < m ^^^ n`, then either `u ^^^ n < m` or `u ^^^ m < n`. obtain ⟨u, rfl⟩ := Ordinal.lt_omega.1 (hu.trans (Ordinal.nat_lt_omega _)) replace hu := Ordinal.nat_cast_lt.1 hu cases' Nat.lt_xor_cases hu with h h -- In the first case, reducing the `m` pile to `u ^^^ n` gives the desired Grundy value. · refine' ⟨toLeftMovesAdd (Sum.inl <| toLeftMovesNim ⟨_, Ordinal.nat_cast_lt.2 h⟩), _⟩ simp [Nat.lxor_cancel_right, hn _ h] -- In the second case, reducing the `n` pile to `u ^^^ m` gives the desired Grundy value. ·
refine' ⟨toLeftMovesAdd (Sum.inr <| toLeftMovesNim ⟨_, Ordinal.nat_cast_lt.2 h⟩), _⟩
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk first | rw [hn _ hk] | rw [hm _ hk] refine' fun h => hk.ne _ rw [Ordinal.nat_cast_inj] at h first | rwa [Nat.xor_left_inj] at h | rwa [Nat.xor_right_inj] at h -- Every other smaller Grundy value can be reached by left moves. · -- If `u < m ^^^ n`, then either `u ^^^ n < m` or `u ^^^ m < n`. obtain ⟨u, rfl⟩ := Ordinal.lt_omega.1 (hu.trans (Ordinal.nat_lt_omega _)) replace hu := Ordinal.nat_cast_lt.1 hu cases' Nat.lt_xor_cases hu with h h -- In the first case, reducing the `m` pile to `u ^^^ n` gives the desired Grundy value. · refine' ⟨toLeftMovesAdd (Sum.inl <| toLeftMovesNim ⟨_, Ordinal.nat_cast_lt.2 h⟩), _⟩ simp [Nat.lxor_cancel_right, hn _ h] -- In the second case, reducing the `n` pile to `u ^^^ m` gives the desired Grundy value. ·
Mathlib.SetTheory.Game.Nim.360_0.mmFMhRYSjViKjcP
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m
Mathlib_SetTheory_Game_Nim
case h.h.refine_2.intro.inr n : ℕ hn : ∀ m < n, ∀ (m_1 : ℕ), grundyValue (nim ↑m + nim ↑m_1) = ↑(m ^^^ m_1) m : ℕ hm : ∀ m_1 < m, grundyValue (nim ↑n + nim ↑m_1) = ↑(n ^^^ m_1) u : ℕ hu : u < n ^^^ m h : u ^^^ n < m ⊢ grundyValue (moveLeft (nim ↑n + nim ↑m) (toLeftMovesAdd (Sum.inr (toLeftMovesNim { val := ↑(u ^^^ n), property := (_ : ↑(u ^^^ n) < ↑m) })))) = ↑u
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq]; exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h⟩ #align pgame.grundy_value_eq_iff_equiv_nim SetTheory.PGame.grundyValue_eq_iff_equiv_nim @[simp] theorem nim_grundyValue (o : Ordinal.{u}) : grundyValue (nim o) = o := grundyValue_eq_iff_equiv_nim.2 PGame.equiv_rfl #align pgame.nim_grundy_value SetTheory.PGame.nim_grundyValue theorem grundyValue_eq_iff_equiv (G H : PGame) [G.Impartial] [H.Impartial] : grundyValue G = grundyValue H ↔ (G ≈ H) := grundyValue_eq_iff_equiv_nim.trans (equiv_congr_left.1 (equiv_nim_grundyValue H) _).symm #align pgame.grundy_value_eq_iff_equiv SetTheory.PGame.grundyValue_eq_iff_equiv @[simp] theorem grundyValue_zero : grundyValue 0 = 0 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_zero_equiv) #align pgame.grundy_value_zero SetTheory.PGame.grundyValue_zero theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by rw [← grundyValue_eq_iff_equiv, grundyValue_zero] #align pgame.grundy_value_iff_equiv_zero SetTheory.PGame.grundyValue_iff_equiv_zero @[simp] theorem grundyValue_star : grundyValue star = 1 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_one_equiv) #align pgame.grundy_value_star SetTheory.PGame.grundyValue_star @[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G := by rw [grundyValue_eq_iff_equiv_nim, neg_equiv_iff, neg_nim, ← grundyValue_eq_iff_equiv_nim] #align pgame.grundy_value_neg SetTheory.PGame.grundyValue_neg theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i haveI : (R i).Impartial := @Impartial.moveRight_impartial ⟨l, r, L, R⟩ _ i apply grundyValue_neg #align pgame.grundy_value_eq_mex_right SetTheory.PGame.grundyValue_eq_mex_right -- Todo: this actually generalizes to all ordinals, by defining `Ordinal.lxor` as the pairwise -- `Nat.xor` of base `ω` Cantor normal forms. /-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk first | rw [hn _ hk] | rw [hm _ hk] refine' fun h => hk.ne _ rw [Ordinal.nat_cast_inj] at h first | rwa [Nat.xor_left_inj] at h | rwa [Nat.xor_right_inj] at h -- Every other smaller Grundy value can be reached by left moves. · -- If `u < m ^^^ n`, then either `u ^^^ n < m` or `u ^^^ m < n`. obtain ⟨u, rfl⟩ := Ordinal.lt_omega.1 (hu.trans (Ordinal.nat_lt_omega _)) replace hu := Ordinal.nat_cast_lt.1 hu cases' Nat.lt_xor_cases hu with h h -- In the first case, reducing the `m` pile to `u ^^^ n` gives the desired Grundy value. · refine' ⟨toLeftMovesAdd (Sum.inl <| toLeftMovesNim ⟨_, Ordinal.nat_cast_lt.2 h⟩), _⟩ simp [Nat.lxor_cancel_right, hn _ h] -- In the second case, reducing the `n` pile to `u ^^^ m` gives the desired Grundy value. · refine' ⟨toLeftMovesAdd (Sum.inr <| toLeftMovesNim ⟨_, Ordinal.nat_cast_lt.2 h⟩), _⟩
have : n ^^^ (u ^^^ n) = u
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk first | rw [hn _ hk] | rw [hm _ hk] refine' fun h => hk.ne _ rw [Ordinal.nat_cast_inj] at h first | rwa [Nat.xor_left_inj] at h | rwa [Nat.xor_right_inj] at h -- Every other smaller Grundy value can be reached by left moves. · -- If `u < m ^^^ n`, then either `u ^^^ n < m` or `u ^^^ m < n`. obtain ⟨u, rfl⟩ := Ordinal.lt_omega.1 (hu.trans (Ordinal.nat_lt_omega _)) replace hu := Ordinal.nat_cast_lt.1 hu cases' Nat.lt_xor_cases hu with h h -- In the first case, reducing the `m` pile to `u ^^^ n` gives the desired Grundy value. · refine' ⟨toLeftMovesAdd (Sum.inl <| toLeftMovesNim ⟨_, Ordinal.nat_cast_lt.2 h⟩), _⟩ simp [Nat.lxor_cancel_right, hn _ h] -- In the second case, reducing the `n` pile to `u ^^^ m` gives the desired Grundy value. · refine' ⟨toLeftMovesAdd (Sum.inr <| toLeftMovesNim ⟨_, Ordinal.nat_cast_lt.2 h⟩), _⟩
Mathlib.SetTheory.Game.Nim.360_0.mmFMhRYSjViKjcP
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m
Mathlib_SetTheory_Game_Nim
case this n : ℕ hn : ∀ m < n, ∀ (m_1 : ℕ), grundyValue (nim ↑m + nim ↑m_1) = ↑(m ^^^ m_1) m : ℕ hm : ∀ m_1 < m, grundyValue (nim ↑n + nim ↑m_1) = ↑(n ^^^ m_1) u : ℕ hu : u < n ^^^ m h : u ^^^ n < m ⊢ n ^^^ (u ^^^ n) = u case h.h.refine_2.intro.inr n : ℕ hn : ∀ m < n, ∀ (m_1 : ℕ), grundyValue (nim ↑m + nim ↑m_1) = ↑(m ^^^ m_1) m : ℕ hm : ∀ m_1 < m, grundyValue (nim ↑n + nim ↑m_1) = ↑(n ^^^ m_1) u : ℕ hu : u < n ^^^ m h : u ^^^ n < m this : n ^^^ (u ^^^ n) = u ⊢ grundyValue (moveLeft (nim ↑n + nim ↑m) (toLeftMovesAdd (Sum.inr (toLeftMovesNim { val := ↑(u ^^^ n), property := (_ : ↑(u ^^^ n) < ↑m) })))) = ↑u
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq]; exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h⟩ #align pgame.grundy_value_eq_iff_equiv_nim SetTheory.PGame.grundyValue_eq_iff_equiv_nim @[simp] theorem nim_grundyValue (o : Ordinal.{u}) : grundyValue (nim o) = o := grundyValue_eq_iff_equiv_nim.2 PGame.equiv_rfl #align pgame.nim_grundy_value SetTheory.PGame.nim_grundyValue theorem grundyValue_eq_iff_equiv (G H : PGame) [G.Impartial] [H.Impartial] : grundyValue G = grundyValue H ↔ (G ≈ H) := grundyValue_eq_iff_equiv_nim.trans (equiv_congr_left.1 (equiv_nim_grundyValue H) _).symm #align pgame.grundy_value_eq_iff_equiv SetTheory.PGame.grundyValue_eq_iff_equiv @[simp] theorem grundyValue_zero : grundyValue 0 = 0 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_zero_equiv) #align pgame.grundy_value_zero SetTheory.PGame.grundyValue_zero theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by rw [← grundyValue_eq_iff_equiv, grundyValue_zero] #align pgame.grundy_value_iff_equiv_zero SetTheory.PGame.grundyValue_iff_equiv_zero @[simp] theorem grundyValue_star : grundyValue star = 1 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_one_equiv) #align pgame.grundy_value_star SetTheory.PGame.grundyValue_star @[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G := by rw [grundyValue_eq_iff_equiv_nim, neg_equiv_iff, neg_nim, ← grundyValue_eq_iff_equiv_nim] #align pgame.grundy_value_neg SetTheory.PGame.grundyValue_neg theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i haveI : (R i).Impartial := @Impartial.moveRight_impartial ⟨l, r, L, R⟩ _ i apply grundyValue_neg #align pgame.grundy_value_eq_mex_right SetTheory.PGame.grundyValue_eq_mex_right -- Todo: this actually generalizes to all ordinals, by defining `Ordinal.lxor` as the pairwise -- `Nat.xor` of base `ω` Cantor normal forms. /-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk first | rw [hn _ hk] | rw [hm _ hk] refine' fun h => hk.ne _ rw [Ordinal.nat_cast_inj] at h first | rwa [Nat.xor_left_inj] at h | rwa [Nat.xor_right_inj] at h -- Every other smaller Grundy value can be reached by left moves. · -- If `u < m ^^^ n`, then either `u ^^^ n < m` or `u ^^^ m < n`. obtain ⟨u, rfl⟩ := Ordinal.lt_omega.1 (hu.trans (Ordinal.nat_lt_omega _)) replace hu := Ordinal.nat_cast_lt.1 hu cases' Nat.lt_xor_cases hu with h h -- In the first case, reducing the `m` pile to `u ^^^ n` gives the desired Grundy value. · refine' ⟨toLeftMovesAdd (Sum.inl <| toLeftMovesNim ⟨_, Ordinal.nat_cast_lt.2 h⟩), _⟩ simp [Nat.lxor_cancel_right, hn _ h] -- In the second case, reducing the `n` pile to `u ^^^ m` gives the desired Grundy value. · refine' ⟨toLeftMovesAdd (Sum.inr <| toLeftMovesNim ⟨_, Ordinal.nat_cast_lt.2 h⟩), _⟩ have : n ^^^ (u ^^^ n) = u;
rw [Nat.xor_comm u, Nat.xor_cancel_left]
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk first | rw [hn _ hk] | rw [hm _ hk] refine' fun h => hk.ne _ rw [Ordinal.nat_cast_inj] at h first | rwa [Nat.xor_left_inj] at h | rwa [Nat.xor_right_inj] at h -- Every other smaller Grundy value can be reached by left moves. · -- If `u < m ^^^ n`, then either `u ^^^ n < m` or `u ^^^ m < n`. obtain ⟨u, rfl⟩ := Ordinal.lt_omega.1 (hu.trans (Ordinal.nat_lt_omega _)) replace hu := Ordinal.nat_cast_lt.1 hu cases' Nat.lt_xor_cases hu with h h -- In the first case, reducing the `m` pile to `u ^^^ n` gives the desired Grundy value. · refine' ⟨toLeftMovesAdd (Sum.inl <| toLeftMovesNim ⟨_, Ordinal.nat_cast_lt.2 h⟩), _⟩ simp [Nat.lxor_cancel_right, hn _ h] -- In the second case, reducing the `n` pile to `u ^^^ m` gives the desired Grundy value. · refine' ⟨toLeftMovesAdd (Sum.inr <| toLeftMovesNim ⟨_, Ordinal.nat_cast_lt.2 h⟩), _⟩ have : n ^^^ (u ^^^ n) = u;
Mathlib.SetTheory.Game.Nim.360_0.mmFMhRYSjViKjcP
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m
Mathlib_SetTheory_Game_Nim
case h.h.refine_2.intro.inr n : ℕ hn : ∀ m < n, ∀ (m_1 : ℕ), grundyValue (nim ↑m + nim ↑m_1) = ↑(m ^^^ m_1) m : ℕ hm : ∀ m_1 < m, grundyValue (nim ↑n + nim ↑m_1) = ↑(n ^^^ m_1) u : ℕ hu : u < n ^^^ m h : u ^^^ n < m this : n ^^^ (u ^^^ n) = u ⊢ grundyValue (moveLeft (nim ↑n + nim ↑m) (toLeftMovesAdd (Sum.inr (toLeftMovesNim { val := ↑(u ^^^ n), property := (_ : ↑(u ^^^ n) < ↑m) })))) = ↑u
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq]; exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h⟩ #align pgame.grundy_value_eq_iff_equiv_nim SetTheory.PGame.grundyValue_eq_iff_equiv_nim @[simp] theorem nim_grundyValue (o : Ordinal.{u}) : grundyValue (nim o) = o := grundyValue_eq_iff_equiv_nim.2 PGame.equiv_rfl #align pgame.nim_grundy_value SetTheory.PGame.nim_grundyValue theorem grundyValue_eq_iff_equiv (G H : PGame) [G.Impartial] [H.Impartial] : grundyValue G = grundyValue H ↔ (G ≈ H) := grundyValue_eq_iff_equiv_nim.trans (equiv_congr_left.1 (equiv_nim_grundyValue H) _).symm #align pgame.grundy_value_eq_iff_equiv SetTheory.PGame.grundyValue_eq_iff_equiv @[simp] theorem grundyValue_zero : grundyValue 0 = 0 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_zero_equiv) #align pgame.grundy_value_zero SetTheory.PGame.grundyValue_zero theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by rw [← grundyValue_eq_iff_equiv, grundyValue_zero] #align pgame.grundy_value_iff_equiv_zero SetTheory.PGame.grundyValue_iff_equiv_zero @[simp] theorem grundyValue_star : grundyValue star = 1 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_one_equiv) #align pgame.grundy_value_star SetTheory.PGame.grundyValue_star @[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G := by rw [grundyValue_eq_iff_equiv_nim, neg_equiv_iff, neg_nim, ← grundyValue_eq_iff_equiv_nim] #align pgame.grundy_value_neg SetTheory.PGame.grundyValue_neg theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i haveI : (R i).Impartial := @Impartial.moveRight_impartial ⟨l, r, L, R⟩ _ i apply grundyValue_neg #align pgame.grundy_value_eq_mex_right SetTheory.PGame.grundyValue_eq_mex_right -- Todo: this actually generalizes to all ordinals, by defining `Ordinal.lxor` as the pairwise -- `Nat.xor` of base `ω` Cantor normal forms. /-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk first | rw [hn _ hk] | rw [hm _ hk] refine' fun h => hk.ne _ rw [Ordinal.nat_cast_inj] at h first | rwa [Nat.xor_left_inj] at h | rwa [Nat.xor_right_inj] at h -- Every other smaller Grundy value can be reached by left moves. · -- If `u < m ^^^ n`, then either `u ^^^ n < m` or `u ^^^ m < n`. obtain ⟨u, rfl⟩ := Ordinal.lt_omega.1 (hu.trans (Ordinal.nat_lt_omega _)) replace hu := Ordinal.nat_cast_lt.1 hu cases' Nat.lt_xor_cases hu with h h -- In the first case, reducing the `m` pile to `u ^^^ n` gives the desired Grundy value. · refine' ⟨toLeftMovesAdd (Sum.inl <| toLeftMovesNim ⟨_, Ordinal.nat_cast_lt.2 h⟩), _⟩ simp [Nat.lxor_cancel_right, hn _ h] -- In the second case, reducing the `n` pile to `u ^^^ m` gives the desired Grundy value. · refine' ⟨toLeftMovesAdd (Sum.inr <| toLeftMovesNim ⟨_, Ordinal.nat_cast_lt.2 h⟩), _⟩ have : n ^^^ (u ^^^ n) = u; rw [Nat.xor_comm u, Nat.xor_cancel_left]
simpa [hm _ h] using this
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk first | rw [hn _ hk] | rw [hm _ hk] refine' fun h => hk.ne _ rw [Ordinal.nat_cast_inj] at h first | rwa [Nat.xor_left_inj] at h | rwa [Nat.xor_right_inj] at h -- Every other smaller Grundy value can be reached by left moves. · -- If `u < m ^^^ n`, then either `u ^^^ n < m` or `u ^^^ m < n`. obtain ⟨u, rfl⟩ := Ordinal.lt_omega.1 (hu.trans (Ordinal.nat_lt_omega _)) replace hu := Ordinal.nat_cast_lt.1 hu cases' Nat.lt_xor_cases hu with h h -- In the first case, reducing the `m` pile to `u ^^^ n` gives the desired Grundy value. · refine' ⟨toLeftMovesAdd (Sum.inl <| toLeftMovesNim ⟨_, Ordinal.nat_cast_lt.2 h⟩), _⟩ simp [Nat.lxor_cancel_right, hn _ h] -- In the second case, reducing the `n` pile to `u ^^^ m` gives the desired Grundy value. · refine' ⟨toLeftMovesAdd (Sum.inr <| toLeftMovesNim ⟨_, Ordinal.nat_cast_lt.2 h⟩), _⟩ have : n ^^^ (u ^^^ n) = u; rw [Nat.xor_comm u, Nat.xor_cancel_left]
Mathlib.SetTheory.Game.Nim.360_0.mmFMhRYSjViKjcP
/-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m
Mathlib_SetTheory_Game_Nim
n m : ℕ ⊢ nim ↑n + nim ↑m ≈ nim ↑(n ^^^ m)
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq]; exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h⟩ #align pgame.grundy_value_eq_iff_equiv_nim SetTheory.PGame.grundyValue_eq_iff_equiv_nim @[simp] theorem nim_grundyValue (o : Ordinal.{u}) : grundyValue (nim o) = o := grundyValue_eq_iff_equiv_nim.2 PGame.equiv_rfl #align pgame.nim_grundy_value SetTheory.PGame.nim_grundyValue theorem grundyValue_eq_iff_equiv (G H : PGame) [G.Impartial] [H.Impartial] : grundyValue G = grundyValue H ↔ (G ≈ H) := grundyValue_eq_iff_equiv_nim.trans (equiv_congr_left.1 (equiv_nim_grundyValue H) _).symm #align pgame.grundy_value_eq_iff_equiv SetTheory.PGame.grundyValue_eq_iff_equiv @[simp] theorem grundyValue_zero : grundyValue 0 = 0 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_zero_equiv) #align pgame.grundy_value_zero SetTheory.PGame.grundyValue_zero theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by rw [← grundyValue_eq_iff_equiv, grundyValue_zero] #align pgame.grundy_value_iff_equiv_zero SetTheory.PGame.grundyValue_iff_equiv_zero @[simp] theorem grundyValue_star : grundyValue star = 1 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_one_equiv) #align pgame.grundy_value_star SetTheory.PGame.grundyValue_star @[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G := by rw [grundyValue_eq_iff_equiv_nim, neg_equiv_iff, neg_nim, ← grundyValue_eq_iff_equiv_nim] #align pgame.grundy_value_neg SetTheory.PGame.grundyValue_neg theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i haveI : (R i).Impartial := @Impartial.moveRight_impartial ⟨l, r, L, R⟩ _ i apply grundyValue_neg #align pgame.grundy_value_eq_mex_right SetTheory.PGame.grundyValue_eq_mex_right -- Todo: this actually generalizes to all ordinals, by defining `Ordinal.lxor` as the pairwise -- `Nat.xor` of base `ω` Cantor normal forms. /-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk first | rw [hn _ hk] | rw [hm _ hk] refine' fun h => hk.ne _ rw [Ordinal.nat_cast_inj] at h first | rwa [Nat.xor_left_inj] at h | rwa [Nat.xor_right_inj] at h -- Every other smaller Grundy value can be reached by left moves. · -- If `u < m ^^^ n`, then either `u ^^^ n < m` or `u ^^^ m < n`. obtain ⟨u, rfl⟩ := Ordinal.lt_omega.1 (hu.trans (Ordinal.nat_lt_omega _)) replace hu := Ordinal.nat_cast_lt.1 hu cases' Nat.lt_xor_cases hu with h h -- In the first case, reducing the `m` pile to `u ^^^ n` gives the desired Grundy value. · refine' ⟨toLeftMovesAdd (Sum.inl <| toLeftMovesNim ⟨_, Ordinal.nat_cast_lt.2 h⟩), _⟩ simp [Nat.lxor_cancel_right, hn _ h] -- In the second case, reducing the `n` pile to `u ^^^ m` gives the desired Grundy value. · refine' ⟨toLeftMovesAdd (Sum.inr <| toLeftMovesNim ⟨_, Ordinal.nat_cast_lt.2 h⟩), _⟩ have : n ^^^ (u ^^^ n) = u; rw [Nat.xor_comm u, Nat.xor_cancel_left] simpa [hm _ h] using this #align pgame.grundy_value_nim_add_nim SetTheory.PGame.grundyValue_nim_add_nim theorem nim_add_nim_equiv {n m : ℕ} : nim n + nim m ≈ nim (n ^^^ m) := by
rw [← grundyValue_eq_iff_equiv_nim, grundyValue_nim_add_nim]
theorem nim_add_nim_equiv {n m : ℕ} : nim n + nim m ≈ nim (n ^^^ m) := by
Mathlib.SetTheory.Game.Nim.402_0.mmFMhRYSjViKjcP
theorem nim_add_nim_equiv {n m : ℕ} : nim n + nim m ≈ nim (n ^^^ m)
Mathlib_SetTheory_Game_Nim
G H : PGame inst✝¹ : Impartial G inst✝ : Impartial H n m : ℕ hG : grundyValue G = ↑n hH : grundyValue H = ↑m ⊢ grundyValue (G + H) = ↑(n ^^^ m)
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq]; exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h⟩ #align pgame.grundy_value_eq_iff_equiv_nim SetTheory.PGame.grundyValue_eq_iff_equiv_nim @[simp] theorem nim_grundyValue (o : Ordinal.{u}) : grundyValue (nim o) = o := grundyValue_eq_iff_equiv_nim.2 PGame.equiv_rfl #align pgame.nim_grundy_value SetTheory.PGame.nim_grundyValue theorem grundyValue_eq_iff_equiv (G H : PGame) [G.Impartial] [H.Impartial] : grundyValue G = grundyValue H ↔ (G ≈ H) := grundyValue_eq_iff_equiv_nim.trans (equiv_congr_left.1 (equiv_nim_grundyValue H) _).symm #align pgame.grundy_value_eq_iff_equiv SetTheory.PGame.grundyValue_eq_iff_equiv @[simp] theorem grundyValue_zero : grundyValue 0 = 0 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_zero_equiv) #align pgame.grundy_value_zero SetTheory.PGame.grundyValue_zero theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by rw [← grundyValue_eq_iff_equiv, grundyValue_zero] #align pgame.grundy_value_iff_equiv_zero SetTheory.PGame.grundyValue_iff_equiv_zero @[simp] theorem grundyValue_star : grundyValue star = 1 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_one_equiv) #align pgame.grundy_value_star SetTheory.PGame.grundyValue_star @[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G := by rw [grundyValue_eq_iff_equiv_nim, neg_equiv_iff, neg_nim, ← grundyValue_eq_iff_equiv_nim] #align pgame.grundy_value_neg SetTheory.PGame.grundyValue_neg theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i haveI : (R i).Impartial := @Impartial.moveRight_impartial ⟨l, r, L, R⟩ _ i apply grundyValue_neg #align pgame.grundy_value_eq_mex_right SetTheory.PGame.grundyValue_eq_mex_right -- Todo: this actually generalizes to all ordinals, by defining `Ordinal.lxor` as the pairwise -- `Nat.xor` of base `ω` Cantor normal forms. /-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk first | rw [hn _ hk] | rw [hm _ hk] refine' fun h => hk.ne _ rw [Ordinal.nat_cast_inj] at h first | rwa [Nat.xor_left_inj] at h | rwa [Nat.xor_right_inj] at h -- Every other smaller Grundy value can be reached by left moves. · -- If `u < m ^^^ n`, then either `u ^^^ n < m` or `u ^^^ m < n`. obtain ⟨u, rfl⟩ := Ordinal.lt_omega.1 (hu.trans (Ordinal.nat_lt_omega _)) replace hu := Ordinal.nat_cast_lt.1 hu cases' Nat.lt_xor_cases hu with h h -- In the first case, reducing the `m` pile to `u ^^^ n` gives the desired Grundy value. · refine' ⟨toLeftMovesAdd (Sum.inl <| toLeftMovesNim ⟨_, Ordinal.nat_cast_lt.2 h⟩), _⟩ simp [Nat.lxor_cancel_right, hn _ h] -- In the second case, reducing the `n` pile to `u ^^^ m` gives the desired Grundy value. · refine' ⟨toLeftMovesAdd (Sum.inr <| toLeftMovesNim ⟨_, Ordinal.nat_cast_lt.2 h⟩), _⟩ have : n ^^^ (u ^^^ n) = u; rw [Nat.xor_comm u, Nat.xor_cancel_left] simpa [hm _ h] using this #align pgame.grundy_value_nim_add_nim SetTheory.PGame.grundyValue_nim_add_nim theorem nim_add_nim_equiv {n m : ℕ} : nim n + nim m ≈ nim (n ^^^ m) := by rw [← grundyValue_eq_iff_equiv_nim, grundyValue_nim_add_nim] #align pgame.nim_add_nim_equiv SetTheory.PGame.nim_add_nim_equiv theorem grundyValue_add (G H : PGame) [G.Impartial] [H.Impartial] {n m : ℕ} (hG : grundyValue G = n) (hH : grundyValue H = m) : grundyValue (G + H) = n ^^^ m := by
rw [← nim_grundyValue (n ^^^ m), grundyValue_eq_iff_equiv]
theorem grundyValue_add (G H : PGame) [G.Impartial] [H.Impartial] {n m : ℕ} (hG : grundyValue G = n) (hH : grundyValue H = m) : grundyValue (G + H) = n ^^^ m := by
Mathlib.SetTheory.Game.Nim.406_0.mmFMhRYSjViKjcP
theorem grundyValue_add (G H : PGame) [G.Impartial] [H.Impartial] {n m : ℕ} (hG : grundyValue G = n) (hH : grundyValue H = m) : grundyValue (G + H) = n ^^^ m
Mathlib_SetTheory_Game_Nim
G H : PGame inst✝¹ : Impartial G inst✝ : Impartial H n m : ℕ hG : grundyValue G = ↑n hH : grundyValue H = ↑m ⊢ G + H ≈ nim ↑(n ^^^ m)
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq]; exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h⟩ #align pgame.grundy_value_eq_iff_equiv_nim SetTheory.PGame.grundyValue_eq_iff_equiv_nim @[simp] theorem nim_grundyValue (o : Ordinal.{u}) : grundyValue (nim o) = o := grundyValue_eq_iff_equiv_nim.2 PGame.equiv_rfl #align pgame.nim_grundy_value SetTheory.PGame.nim_grundyValue theorem grundyValue_eq_iff_equiv (G H : PGame) [G.Impartial] [H.Impartial] : grundyValue G = grundyValue H ↔ (G ≈ H) := grundyValue_eq_iff_equiv_nim.trans (equiv_congr_left.1 (equiv_nim_grundyValue H) _).symm #align pgame.grundy_value_eq_iff_equiv SetTheory.PGame.grundyValue_eq_iff_equiv @[simp] theorem grundyValue_zero : grundyValue 0 = 0 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_zero_equiv) #align pgame.grundy_value_zero SetTheory.PGame.grundyValue_zero theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by rw [← grundyValue_eq_iff_equiv, grundyValue_zero] #align pgame.grundy_value_iff_equiv_zero SetTheory.PGame.grundyValue_iff_equiv_zero @[simp] theorem grundyValue_star : grundyValue star = 1 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_one_equiv) #align pgame.grundy_value_star SetTheory.PGame.grundyValue_star @[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G := by rw [grundyValue_eq_iff_equiv_nim, neg_equiv_iff, neg_nim, ← grundyValue_eq_iff_equiv_nim] #align pgame.grundy_value_neg SetTheory.PGame.grundyValue_neg theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i haveI : (R i).Impartial := @Impartial.moveRight_impartial ⟨l, r, L, R⟩ _ i apply grundyValue_neg #align pgame.grundy_value_eq_mex_right SetTheory.PGame.grundyValue_eq_mex_right -- Todo: this actually generalizes to all ordinals, by defining `Ordinal.lxor` as the pairwise -- `Nat.xor` of base `ω` Cantor normal forms. /-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk first | rw [hn _ hk] | rw [hm _ hk] refine' fun h => hk.ne _ rw [Ordinal.nat_cast_inj] at h first | rwa [Nat.xor_left_inj] at h | rwa [Nat.xor_right_inj] at h -- Every other smaller Grundy value can be reached by left moves. · -- If `u < m ^^^ n`, then either `u ^^^ n < m` or `u ^^^ m < n`. obtain ⟨u, rfl⟩ := Ordinal.lt_omega.1 (hu.trans (Ordinal.nat_lt_omega _)) replace hu := Ordinal.nat_cast_lt.1 hu cases' Nat.lt_xor_cases hu with h h -- In the first case, reducing the `m` pile to `u ^^^ n` gives the desired Grundy value. · refine' ⟨toLeftMovesAdd (Sum.inl <| toLeftMovesNim ⟨_, Ordinal.nat_cast_lt.2 h⟩), _⟩ simp [Nat.lxor_cancel_right, hn _ h] -- In the second case, reducing the `n` pile to `u ^^^ m` gives the desired Grundy value. · refine' ⟨toLeftMovesAdd (Sum.inr <| toLeftMovesNim ⟨_, Ordinal.nat_cast_lt.2 h⟩), _⟩ have : n ^^^ (u ^^^ n) = u; rw [Nat.xor_comm u, Nat.xor_cancel_left] simpa [hm _ h] using this #align pgame.grundy_value_nim_add_nim SetTheory.PGame.grundyValue_nim_add_nim theorem nim_add_nim_equiv {n m : ℕ} : nim n + nim m ≈ nim (n ^^^ m) := by rw [← grundyValue_eq_iff_equiv_nim, grundyValue_nim_add_nim] #align pgame.nim_add_nim_equiv SetTheory.PGame.nim_add_nim_equiv theorem grundyValue_add (G H : PGame) [G.Impartial] [H.Impartial] {n m : ℕ} (hG : grundyValue G = n) (hH : grundyValue H = m) : grundyValue (G + H) = n ^^^ m := by rw [← nim_grundyValue (n ^^^ m), grundyValue_eq_iff_equiv]
refine' Equiv.trans _ nim_add_nim_equiv
theorem grundyValue_add (G H : PGame) [G.Impartial] [H.Impartial] {n m : ℕ} (hG : grundyValue G = n) (hH : grundyValue H = m) : grundyValue (G + H) = n ^^^ m := by rw [← nim_grundyValue (n ^^^ m), grundyValue_eq_iff_equiv]
Mathlib.SetTheory.Game.Nim.406_0.mmFMhRYSjViKjcP
theorem grundyValue_add (G H : PGame) [G.Impartial] [H.Impartial] {n m : ℕ} (hG : grundyValue G = n) (hH : grundyValue H = m) : grundyValue (G + H) = n ^^^ m
Mathlib_SetTheory_Game_Nim
G H : PGame inst✝¹ : Impartial G inst✝ : Impartial H n m : ℕ hG : grundyValue G = ↑n hH : grundyValue H = ↑m ⊢ G + H ≈ nim ↑n + nim ↑m
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq]; exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h⟩ #align pgame.grundy_value_eq_iff_equiv_nim SetTheory.PGame.grundyValue_eq_iff_equiv_nim @[simp] theorem nim_grundyValue (o : Ordinal.{u}) : grundyValue (nim o) = o := grundyValue_eq_iff_equiv_nim.2 PGame.equiv_rfl #align pgame.nim_grundy_value SetTheory.PGame.nim_grundyValue theorem grundyValue_eq_iff_equiv (G H : PGame) [G.Impartial] [H.Impartial] : grundyValue G = grundyValue H ↔ (G ≈ H) := grundyValue_eq_iff_equiv_nim.trans (equiv_congr_left.1 (equiv_nim_grundyValue H) _).symm #align pgame.grundy_value_eq_iff_equiv SetTheory.PGame.grundyValue_eq_iff_equiv @[simp] theorem grundyValue_zero : grundyValue 0 = 0 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_zero_equiv) #align pgame.grundy_value_zero SetTheory.PGame.grundyValue_zero theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by rw [← grundyValue_eq_iff_equiv, grundyValue_zero] #align pgame.grundy_value_iff_equiv_zero SetTheory.PGame.grundyValue_iff_equiv_zero @[simp] theorem grundyValue_star : grundyValue star = 1 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_one_equiv) #align pgame.grundy_value_star SetTheory.PGame.grundyValue_star @[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G := by rw [grundyValue_eq_iff_equiv_nim, neg_equiv_iff, neg_nim, ← grundyValue_eq_iff_equiv_nim] #align pgame.grundy_value_neg SetTheory.PGame.grundyValue_neg theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i haveI : (R i).Impartial := @Impartial.moveRight_impartial ⟨l, r, L, R⟩ _ i apply grundyValue_neg #align pgame.grundy_value_eq_mex_right SetTheory.PGame.grundyValue_eq_mex_right -- Todo: this actually generalizes to all ordinals, by defining `Ordinal.lxor` as the pairwise -- `Nat.xor` of base `ω` Cantor normal forms. /-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk first | rw [hn _ hk] | rw [hm _ hk] refine' fun h => hk.ne _ rw [Ordinal.nat_cast_inj] at h first | rwa [Nat.xor_left_inj] at h | rwa [Nat.xor_right_inj] at h -- Every other smaller Grundy value can be reached by left moves. · -- If `u < m ^^^ n`, then either `u ^^^ n < m` or `u ^^^ m < n`. obtain ⟨u, rfl⟩ := Ordinal.lt_omega.1 (hu.trans (Ordinal.nat_lt_omega _)) replace hu := Ordinal.nat_cast_lt.1 hu cases' Nat.lt_xor_cases hu with h h -- In the first case, reducing the `m` pile to `u ^^^ n` gives the desired Grundy value. · refine' ⟨toLeftMovesAdd (Sum.inl <| toLeftMovesNim ⟨_, Ordinal.nat_cast_lt.2 h⟩), _⟩ simp [Nat.lxor_cancel_right, hn _ h] -- In the second case, reducing the `n` pile to `u ^^^ m` gives the desired Grundy value. · refine' ⟨toLeftMovesAdd (Sum.inr <| toLeftMovesNim ⟨_, Ordinal.nat_cast_lt.2 h⟩), _⟩ have : n ^^^ (u ^^^ n) = u; rw [Nat.xor_comm u, Nat.xor_cancel_left] simpa [hm _ h] using this #align pgame.grundy_value_nim_add_nim SetTheory.PGame.grundyValue_nim_add_nim theorem nim_add_nim_equiv {n m : ℕ} : nim n + nim m ≈ nim (n ^^^ m) := by rw [← grundyValue_eq_iff_equiv_nim, grundyValue_nim_add_nim] #align pgame.nim_add_nim_equiv SetTheory.PGame.nim_add_nim_equiv theorem grundyValue_add (G H : PGame) [G.Impartial] [H.Impartial] {n m : ℕ} (hG : grundyValue G = n) (hH : grundyValue H = m) : grundyValue (G + H) = n ^^^ m := by rw [← nim_grundyValue (n ^^^ m), grundyValue_eq_iff_equiv] refine' Equiv.trans _ nim_add_nim_equiv
convert add_congr (equiv_nim_grundyValue G) (equiv_nim_grundyValue H)
theorem grundyValue_add (G H : PGame) [G.Impartial] [H.Impartial] {n m : ℕ} (hG : grundyValue G = n) (hH : grundyValue H = m) : grundyValue (G + H) = n ^^^ m := by rw [← nim_grundyValue (n ^^^ m), grundyValue_eq_iff_equiv] refine' Equiv.trans _ nim_add_nim_equiv
Mathlib.SetTheory.Game.Nim.406_0.mmFMhRYSjViKjcP
theorem grundyValue_add (G H : PGame) [G.Impartial] [H.Impartial] {n m : ℕ} (hG : grundyValue G = n) (hH : grundyValue H = m) : grundyValue (G + H) = n ^^^ m
Mathlib_SetTheory_Game_Nim
case h.e'_4.h.e'_5.h.e'_1 G H : PGame inst✝¹ : Impartial G inst✝ : Impartial H n m : ℕ hG : grundyValue G = ↑n hH : grundyValue H = ↑m ⊢ ↑n = grundyValue G
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq]; exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h⟩ #align pgame.grundy_value_eq_iff_equiv_nim SetTheory.PGame.grundyValue_eq_iff_equiv_nim @[simp] theorem nim_grundyValue (o : Ordinal.{u}) : grundyValue (nim o) = o := grundyValue_eq_iff_equiv_nim.2 PGame.equiv_rfl #align pgame.nim_grundy_value SetTheory.PGame.nim_grundyValue theorem grundyValue_eq_iff_equiv (G H : PGame) [G.Impartial] [H.Impartial] : grundyValue G = grundyValue H ↔ (G ≈ H) := grundyValue_eq_iff_equiv_nim.trans (equiv_congr_left.1 (equiv_nim_grundyValue H) _).symm #align pgame.grundy_value_eq_iff_equiv SetTheory.PGame.grundyValue_eq_iff_equiv @[simp] theorem grundyValue_zero : grundyValue 0 = 0 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_zero_equiv) #align pgame.grundy_value_zero SetTheory.PGame.grundyValue_zero theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by rw [← grundyValue_eq_iff_equiv, grundyValue_zero] #align pgame.grundy_value_iff_equiv_zero SetTheory.PGame.grundyValue_iff_equiv_zero @[simp] theorem grundyValue_star : grundyValue star = 1 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_one_equiv) #align pgame.grundy_value_star SetTheory.PGame.grundyValue_star @[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G := by rw [grundyValue_eq_iff_equiv_nim, neg_equiv_iff, neg_nim, ← grundyValue_eq_iff_equiv_nim] #align pgame.grundy_value_neg SetTheory.PGame.grundyValue_neg theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i haveI : (R i).Impartial := @Impartial.moveRight_impartial ⟨l, r, L, R⟩ _ i apply grundyValue_neg #align pgame.grundy_value_eq_mex_right SetTheory.PGame.grundyValue_eq_mex_right -- Todo: this actually generalizes to all ordinals, by defining `Ordinal.lxor` as the pairwise -- `Nat.xor` of base `ω` Cantor normal forms. /-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk first | rw [hn _ hk] | rw [hm _ hk] refine' fun h => hk.ne _ rw [Ordinal.nat_cast_inj] at h first | rwa [Nat.xor_left_inj] at h | rwa [Nat.xor_right_inj] at h -- Every other smaller Grundy value can be reached by left moves. · -- If `u < m ^^^ n`, then either `u ^^^ n < m` or `u ^^^ m < n`. obtain ⟨u, rfl⟩ := Ordinal.lt_omega.1 (hu.trans (Ordinal.nat_lt_omega _)) replace hu := Ordinal.nat_cast_lt.1 hu cases' Nat.lt_xor_cases hu with h h -- In the first case, reducing the `m` pile to `u ^^^ n` gives the desired Grundy value. · refine' ⟨toLeftMovesAdd (Sum.inl <| toLeftMovesNim ⟨_, Ordinal.nat_cast_lt.2 h⟩), _⟩ simp [Nat.lxor_cancel_right, hn _ h] -- In the second case, reducing the `n` pile to `u ^^^ m` gives the desired Grundy value. · refine' ⟨toLeftMovesAdd (Sum.inr <| toLeftMovesNim ⟨_, Ordinal.nat_cast_lt.2 h⟩), _⟩ have : n ^^^ (u ^^^ n) = u; rw [Nat.xor_comm u, Nat.xor_cancel_left] simpa [hm _ h] using this #align pgame.grundy_value_nim_add_nim SetTheory.PGame.grundyValue_nim_add_nim theorem nim_add_nim_equiv {n m : ℕ} : nim n + nim m ≈ nim (n ^^^ m) := by rw [← grundyValue_eq_iff_equiv_nim, grundyValue_nim_add_nim] #align pgame.nim_add_nim_equiv SetTheory.PGame.nim_add_nim_equiv theorem grundyValue_add (G H : PGame) [G.Impartial] [H.Impartial] {n m : ℕ} (hG : grundyValue G = n) (hH : grundyValue H = m) : grundyValue (G + H) = n ^^^ m := by rw [← nim_grundyValue (n ^^^ m), grundyValue_eq_iff_equiv] refine' Equiv.trans _ nim_add_nim_equiv convert add_congr (equiv_nim_grundyValue G) (equiv_nim_grundyValue H) <;>
simp only [hG, hH]
theorem grundyValue_add (G H : PGame) [G.Impartial] [H.Impartial] {n m : ℕ} (hG : grundyValue G = n) (hH : grundyValue H = m) : grundyValue (G + H) = n ^^^ m := by rw [← nim_grundyValue (n ^^^ m), grundyValue_eq_iff_equiv] refine' Equiv.trans _ nim_add_nim_equiv convert add_congr (equiv_nim_grundyValue G) (equiv_nim_grundyValue H) <;>
Mathlib.SetTheory.Game.Nim.406_0.mmFMhRYSjViKjcP
theorem grundyValue_add (G H : PGame) [G.Impartial] [H.Impartial] {n m : ℕ} (hG : grundyValue G = n) (hH : grundyValue H = m) : grundyValue (G + H) = n ^^^ m
Mathlib_SetTheory_Game_Nim
case h.e'_4.h.e'_6.h.e'_1 G H : PGame inst✝¹ : Impartial G inst✝ : Impartial H n m : ℕ hG : grundyValue G = ↑n hH : grundyValue H = ↑m ⊢ ↑m = grundyValue H
/- Copyright (c) 2020 Fox Thomson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Fox Thomson, Markus Himmel -/ import Mathlib.Data.Nat.Bitwise import Mathlib.SetTheory.Game.Birthday import Mathlib.SetTheory.Game.Impartial #align_import set_theory.game.nim from "leanprover-community/mathlib"@"92ca63f0fb391a9ca5f22d2409a6080e786d99f7" /-! # Nim and the Sprague-Grundy theorem This file contains the definition for nim for any ordinal `o`. In the game of `nim o₁` both players may move to `nim o₂` for any `o₂ < o₁`. We also define a Grundy value for an impartial game `G` and prove the Sprague-Grundy theorem, that `G` is equivalent to `nim (grundyValue G)`. Finally, we compute the sum of finite Grundy numbers: if `G` and `H` have Grundy values `n` and `m`, where `n` and `m` are natural numbers, then `G + H` has the Grundy value `n xor m`. ## Implementation details The pen-and-paper definition of nim defines the possible moves of `nim o` to be `Set.Iio o`. However, this definition does not work for us because it would make the type of nim `Ordinal.{u} → SetTheory.PGame.{u + 1}`, which would make it impossible for us to state the Sprague-Grundy theorem, since that requires the type of `nim` to be `Ordinal.{u} → SetTheory.PGame.{u}`. For this reason, we instead use `o.out.α` for the possible moves. You can use `to_left_moves_nim` and `to_right_moves_nim` to convert an ordinal less than `o` into a left or right move of `nim o`, and vice versa. -/ noncomputable section universe u namespace SetTheory open scoped PGame namespace PGame -- Uses `noncomputable!` to avoid `rec_fn_macro only allowed in meta definitions` VM error /-- The definition of single-heap nim, which can be viewed as a pile of stones where each player can take a positive number of stones from it on their turn. -/ noncomputable def nim : Ordinal.{u} → PGame.{u} | o₁ => let f o₂ := have _ : Ordinal.typein o₁.out.r o₂ < o₁ := Ordinal.typein_lt_self o₂ nim (Ordinal.typein o₁.out.r o₂) ⟨o₁.out.α, o₁.out.α, f, f⟩ termination_by nim o => o #align pgame.nim SetTheory.PGame.nim open Ordinal theorem nim_def (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance nim o = PGame.mk o.out.α o.out.α (fun o₂ => nim (Ordinal.typein (· < ·) o₂)) fun o₂ => nim (Ordinal.typein (· < ·) o₂) := by rw [nim]; rfl #align pgame.nim_def SetTheory.PGame.nim_def theorem leftMoves_nim (o : Ordinal) : (nim o).LeftMoves = o.out.α := by rw [nim_def]; rfl #align pgame.left_moves_nim SetTheory.PGame.leftMoves_nim theorem rightMoves_nim (o : Ordinal) : (nim o).RightMoves = o.out.α := by rw [nim_def]; rfl #align pgame.right_moves_nim SetTheory.PGame.rightMoves_nim theorem moveLeft_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveLeft fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_left_nim_heq SetTheory.PGame.moveLeft_nim_hEq theorem moveRight_nim_hEq (o : Ordinal) : have : IsWellOrder (Quotient.out o).α (· < ·) := inferInstance HEq (nim o).moveRight fun i : o.out.α => nim (typein (· < ·) i) := by rw [nim_def]; rfl #align pgame.move_right_nim_heq SetTheory.PGame.moveRight_nim_hEq /-- Turns an ordinal less than `o` into a left move for `nim o` and viceversa. -/ noncomputable def toLeftMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).LeftMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (leftMoves_nim o).symm) #align pgame.to_left_moves_nim SetTheory.PGame.toLeftMovesNim /-- Turns an ordinal less than `o` into a right move for `nim o` and viceversa. -/ noncomputable def toRightMovesNim {o : Ordinal} : Set.Iio o ≃ (nim o).RightMoves := (enumIsoOut o).toEquiv.trans (Equiv.cast (rightMoves_nim o).symm) #align pgame.to_right_moves_nim SetTheory.PGame.toRightMovesNim @[simp] theorem toLeftMovesNim_symm_lt {o : Ordinal} (i : (nim o).LeftMoves) : ↑(toLeftMovesNim.symm i) < o := (toLeftMovesNim.symm i).prop #align pgame.to_left_moves_nim_symm_lt SetTheory.PGame.toLeftMovesNim_symm_lt @[simp] theorem toRightMovesNim_symm_lt {o : Ordinal} (i : (nim o).RightMoves) : ↑(toRightMovesNim.symm i) < o := (toRightMovesNim.symm i).prop #align pgame.to_right_moves_nim_symm_lt SetTheory.PGame.toRightMovesNim_symm_lt @[simp] theorem moveLeft_nim' {o : Ordinal.{u}} (i) : (nim o).moveLeft i = nim (toLeftMovesNim.symm i).val := (congr_heq (moveLeft_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_left_nim' SetTheory.PGame.moveLeft_nim' theorem moveLeft_nim {o : Ordinal} (i) : (nim o).moveLeft (toLeftMovesNim i) = nim i := by simp #align pgame.move_left_nim SetTheory.PGame.moveLeft_nim @[simp] theorem moveRight_nim' {o : Ordinal} (i) : (nim o).moveRight i = nim (toRightMovesNim.symm i).val := (congr_heq (moveRight_nim_hEq o).symm (cast_heq _ i)).symm #align pgame.move_right_nim' SetTheory.PGame.moveRight_nim' theorem moveRight_nim {o : Ordinal} (i) : (nim o).moveRight (toRightMovesNim i) = nim i := by simp #align pgame.move_right_nim SetTheory.PGame.moveRight_nim /-- A recursion principle for left moves of a nim game. -/ @[elab_as_elim] def leftMovesNimRecOn {o : Ordinal} {P : (nim o).LeftMoves → Sort*} (i : (nim o).LeftMoves) (H : ∀ a (H : a < o), P <| toLeftMovesNim ⟨a, H⟩) : P i := by rw [← toLeftMovesNim.apply_symm_apply i]; apply H #align pgame.left_moves_nim_rec_on SetTheory.PGame.leftMovesNimRecOn /-- A recursion principle for right moves of a nim game. -/ @[elab_as_elim] def rightMovesNimRecOn {o : Ordinal} {P : (nim o).RightMoves → Sort*} (i : (nim o).RightMoves) (H : ∀ a (H : a < o), P <| toRightMovesNim ⟨a, H⟩) : P i := by rw [← toRightMovesNim.apply_symm_apply i]; apply H #align pgame.right_moves_nim_rec_on SetTheory.PGame.rightMovesNimRecOn instance isEmpty_nim_zero_leftMoves : IsEmpty (nim 0).LeftMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_left_moves SetTheory.PGame.isEmpty_nim_zero_leftMoves instance isEmpty_nim_zero_rightMoves : IsEmpty (nim 0).RightMoves := by rw [nim_def] exact Ordinal.isEmpty_out_zero #align pgame.is_empty_nim_zero_right_moves SetTheory.PGame.isEmpty_nim_zero_rightMoves /-- `nim 0` has exactly the same moves as `0`. -/ def nimZeroRelabelling : nim 0 ≡r 0 := Relabelling.isEmpty _ #align pgame.nim_zero_relabelling SetTheory.PGame.nimZeroRelabelling theorem nim_zero_equiv : nim 0 ≈ 0 := Equiv.isEmpty _ #align pgame.nim_zero_equiv SetTheory.PGame.nim_zero_equiv noncomputable instance uniqueNimOneLeftMoves : Unique (nim 1).LeftMoves := (Equiv.cast <| leftMoves_nim 1).unique #align pgame.unique_nim_one_left_moves SetTheory.PGame.uniqueNimOneLeftMoves noncomputable instance uniqueNimOneRightMoves : Unique (nim 1).RightMoves := (Equiv.cast <| rightMoves_nim 1).unique #align pgame.unique_nim_one_right_moves SetTheory.PGame.uniqueNimOneRightMoves @[simp] theorem default_nim_one_leftMoves_eq : (default : (nim 1).LeftMoves) = @toLeftMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_left_moves_eq SetTheory.PGame.default_nim_one_leftMoves_eq @[simp] theorem default_nim_one_rightMoves_eq : (default : (nim 1).RightMoves) = @toRightMovesNim 1 ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := rfl #align pgame.default_nim_one_right_moves_eq SetTheory.PGame.default_nim_one_rightMoves_eq @[simp] theorem toLeftMovesNim_one_symm (i) : (@toLeftMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_left_moves_nim_one_symm SetTheory.PGame.toLeftMovesNim_one_symm @[simp] theorem toRightMovesNim_one_symm (i) : (@toRightMovesNim 1).symm i = ⟨0, Set.mem_Iio.mpr zero_lt_one⟩ := by simp [eq_iff_true_of_subsingleton] #align pgame.to_right_moves_nim_one_symm SetTheory.PGame.toRightMovesNim_one_symm theorem nim_one_moveLeft (x) : (nim 1).moveLeft x = nim 0 := by simp #align pgame.nim_one_move_left SetTheory.PGame.nim_one_moveLeft theorem nim_one_moveRight (x) : (nim 1).moveRight x = nim 0 := by simp #align pgame.nim_one_move_right SetTheory.PGame.nim_one_moveRight /-- `nim 1` has exactly the same moves as `star`. -/ def nimOneRelabelling : nim 1 ≡r star := by rw [nim_def] refine' ⟨_, _, fun i => _, fun j => _⟩ any_goals dsimp; apply Equiv.equivOfUnique all_goals simp; exact nimZeroRelabelling #align pgame.nim_one_relabelling SetTheory.PGame.nimOneRelabelling theorem nim_one_equiv : nim 1 ≈ star := nimOneRelabelling.equiv #align pgame.nim_one_equiv SetTheory.PGame.nim_one_equiv @[simp] theorem nim_birthday (o : Ordinal) : (nim o).birthday = o := by induction' o using Ordinal.induction with o IH rw [nim_def, birthday_def] dsimp rw [max_eq_right le_rfl] convert lsub_typein o with i exact IH _ (typein_lt_self i) #align pgame.nim_birthday SetTheory.PGame.nim_birthday @[simp] theorem neg_nim (o : Ordinal) : -nim o = nim o := by induction' o using Ordinal.induction with o IH rw [nim_def]; dsimp; congr <;> funext i <;> exact IH _ (Ordinal.typein_lt_self i) #align pgame.neg_nim SetTheory.PGame.neg_nim instance nim_impartial (o : Ordinal) : Impartial (nim o) := by induction' o using Ordinal.induction with o IH rw [impartial_def, neg_nim] refine' ⟨equiv_rfl, fun i => _, fun i => _⟩ <;> simpa using IH _ (typein_lt_self _) #align pgame.nim_impartial SetTheory.PGame.nim_impartial theorem nim_fuzzy_zero_of_ne_zero {o : Ordinal} (ho : o ≠ 0) : nim o ‖ 0 := by rw [Impartial.fuzzy_zero_iff_lf, nim_def, lf_zero_le] rw [← Ordinal.pos_iff_ne_zero] at ho exact ⟨(Ordinal.principalSegOut ho).top, by simp⟩ #align pgame.nim_fuzzy_zero_of_ne_zero SetTheory.PGame.nim_fuzzy_zero_of_ne_zero @[simp] theorem nim_add_equiv_zero_iff (o₁ o₂ : Ordinal) : (nim o₁ + nim o₂ ≈ 0) ↔ o₁ = o₂ := by constructor · refine' not_imp_not.1 fun hne : _ ≠ _ => (Impartial.not_equiv_zero_iff (nim o₁ + nim o₂)).2 _ wlog h : o₁ < o₂ · exact (fuzzy_congr_left add_comm_equiv).1 (this _ _ hne.symm (hne.lt_or_lt.resolve_left h)) rw [Impartial.fuzzy_zero_iff_gf, zero_lf_le, nim_def o₂] refine' ⟨toLeftMovesAdd (Sum.inr _), _⟩ · exact (Ordinal.principalSegOut h).top · -- Porting note: squeezed simp simpa only [Ordinal.typein_top, Ordinal.type_lt, PGame.add_moveLeft_inr, PGame.moveLeft_mk] using (Impartial.add_self (nim o₁)).2 · rintro rfl exact Impartial.add_self (nim o₁) #align pgame.nim_add_equiv_zero_iff SetTheory.PGame.nim_add_equiv_zero_iff @[simp] theorem nim_add_fuzzy_zero_iff {o₁ o₂ : Ordinal} : nim o₁ + nim o₂ ‖ 0 ↔ o₁ ≠ o₂ := by rw [iff_not_comm, Impartial.not_fuzzy_zero_iff, nim_add_equiv_zero_iff] #align pgame.nim_add_fuzzy_zero_iff SetTheory.PGame.nim_add_fuzzy_zero_iff @[simp] theorem nim_equiv_iff_eq {o₁ o₂ : Ordinal} : (nim o₁ ≈ nim o₂) ↔ o₁ = o₂ := by rw [Impartial.equiv_iff_add_equiv_zero, nim_add_equiv_zero_iff] #align pgame.nim_equiv_iff_eq SetTheory.PGame.nim_equiv_iff_eq /-- The Grundy value of an impartial game, the ordinal which corresponds to the game of nim that the game is equivalent to -/ noncomputable def grundyValue : ∀ _ : PGame.{u}, Ordinal.{u} | G => Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) termination_by grundyValue G => G decreasing_by pgame_wf_tac #align pgame.grundy_value SetTheory.PGame.grundyValue theorem grundyValue_eq_mex_left (G : PGame) : grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveLeft i) := by rw [grundyValue] #align pgame.grundy_value_eq_mex_left SetTheory.PGame.grundyValue_eq_mex_left /-- The Sprague-Grundy theorem which states that every impartial game is equivalent to a game of nim, namely the game of nim corresponding to the games Grundy value -/ theorem equiv_nim_grundyValue : ∀ (G : PGame.{u}) [G.Impartial], G ≈ nim (grundyValue G) | G => by rw [Impartial.equiv_iff_add_equiv_zero, ← Impartial.forall_leftMoves_fuzzy_iff_equiv_zero] intro i apply leftMoves_add_cases i · intro i₁ rw [add_moveLeft_inl] apply (fuzzy_congr_left (add_congr_left (Equiv.symm (equiv_nim_grundyValue (G.moveLeft i₁))))).1 rw [nim_add_fuzzy_zero_iff] intro heq rw [eq_comm, grundyValue_eq_mex_left G] at heq -- Porting note: added universe annotation, argument have h := Ordinal.ne_mex.{u, u} (fun i ↦ grundyValue (moveLeft G i)) rw [heq] at h exact (h i₁).irrefl · intro i₂ rw [add_moveLeft_inr, ← Impartial.exists_left_move_equiv_iff_fuzzy_zero] revert i₂ rw [nim_def] intro i₂ have h' : ∃ i : G.LeftMoves, grundyValue (G.moveLeft i) = Ordinal.typein (Quotient.out (grundyValue G)).r i₂ := by revert i₂ rw [grundyValue_eq_mex_left] intro i₂ have hnotin : _ ∉ _ := fun hin => (le_not_le_of_lt (Ordinal.typein_lt_self i₂)).2 (csInf_le' hin) simpa using hnotin cases' h' with i hi use toLeftMovesAdd (Sum.inl i) rw [add_moveLeft_inl, moveLeft_mk] apply Equiv.trans (add_congr_left (equiv_nim_grundyValue (G.moveLeft i))) simpa only [hi] using Impartial.add_self (nim (grundyValue (G.moveLeft i))) termination_by equiv_nim_grundyValue G _ => G decreasing_by pgame_wf_tac #align pgame.equiv_nim_grundy_value SetTheory.PGame.equiv_nim_grundyValue theorem grundyValue_eq_iff_equiv_nim {G : PGame} [G.Impartial] {o : Ordinal} : grundyValue G = o ↔ (G ≈ nim o) := ⟨by rintro rfl; exact equiv_nim_grundyValue G, by intro h; rw [← nim_equiv_iff_eq]; exact Equiv.trans (Equiv.symm (equiv_nim_grundyValue G)) h⟩ #align pgame.grundy_value_eq_iff_equiv_nim SetTheory.PGame.grundyValue_eq_iff_equiv_nim @[simp] theorem nim_grundyValue (o : Ordinal.{u}) : grundyValue (nim o) = o := grundyValue_eq_iff_equiv_nim.2 PGame.equiv_rfl #align pgame.nim_grundy_value SetTheory.PGame.nim_grundyValue theorem grundyValue_eq_iff_equiv (G H : PGame) [G.Impartial] [H.Impartial] : grundyValue G = grundyValue H ↔ (G ≈ H) := grundyValue_eq_iff_equiv_nim.trans (equiv_congr_left.1 (equiv_nim_grundyValue H) _).symm #align pgame.grundy_value_eq_iff_equiv SetTheory.PGame.grundyValue_eq_iff_equiv @[simp] theorem grundyValue_zero : grundyValue 0 = 0 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_zero_equiv) #align pgame.grundy_value_zero SetTheory.PGame.grundyValue_zero theorem grundyValue_iff_equiv_zero (G : PGame) [G.Impartial] : grundyValue G = 0 ↔ (G ≈ 0) := by rw [← grundyValue_eq_iff_equiv, grundyValue_zero] #align pgame.grundy_value_iff_equiv_zero SetTheory.PGame.grundyValue_iff_equiv_zero @[simp] theorem grundyValue_star : grundyValue star = 1 := grundyValue_eq_iff_equiv_nim.2 (Equiv.symm nim_one_equiv) #align pgame.grundy_value_star SetTheory.PGame.grundyValue_star @[simp] theorem grundyValue_neg (G : PGame) [G.Impartial] : grundyValue (-G) = grundyValue G := by rw [grundyValue_eq_iff_equiv_nim, neg_equiv_iff, neg_nim, ← grundyValue_eq_iff_equiv_nim] #align pgame.grundy_value_neg SetTheory.PGame.grundyValue_neg theorem grundyValue_eq_mex_right : ∀ (G : PGame) [G.Impartial], grundyValue G = Ordinal.mex.{u, u} fun i => grundyValue (G.moveRight i) | ⟨l, r, L, R⟩, _ => by rw [← grundyValue_neg, grundyValue_eq_mex_left] congr ext i haveI : (R i).Impartial := @Impartial.moveRight_impartial ⟨l, r, L, R⟩ _ i apply grundyValue_neg #align pgame.grundy_value_eq_mex_right SetTheory.PGame.grundyValue_eq_mex_right -- Todo: this actually generalizes to all ordinals, by defining `Ordinal.lxor` as the pairwise -- `Nat.xor` of base `ω` Cantor normal forms. /-- The Grundy value of the sum of two nim games with natural numbers of piles equals their bitwise xor. -/ @[simp] theorem grundyValue_nim_add_nim (n m : ℕ) : grundyValue (nim.{u} n + nim.{u} m) = n ^^^ m := by -- We do strong induction on both variables. induction' n using Nat.strong_induction_on with n hn generalizing m induction' m using Nat.strong_induction_on with m hm rw [grundyValue_eq_mex_left] refine (Ordinal.mex_le_of_ne.{u, u} fun i => ?_).antisymm (Ordinal.le_mex_of_forall fun ou hu => ?_) -- The Grundy value `n ^^^ m` can't be reached by left moves. · apply leftMoves_add_cases i <;> · -- A left move leaves us with a Grundy value of `k ^^^ m` for `k < n`, or -- `n ^^^ k` for `k < m`. refine' fun a => leftMovesNimRecOn a fun ok hk => _ obtain ⟨k, rfl⟩ := Ordinal.lt_omega.1 (hk.trans (Ordinal.nat_lt_omega _)) simp only [add_moveLeft_inl, add_moveLeft_inr, moveLeft_nim', Equiv.symm_apply_apply] -- The inequality follows from injectivity. rw [nat_cast_lt] at hk first | rw [hn _ hk] | rw [hm _ hk] refine' fun h => hk.ne _ rw [Ordinal.nat_cast_inj] at h first | rwa [Nat.xor_left_inj] at h | rwa [Nat.xor_right_inj] at h -- Every other smaller Grundy value can be reached by left moves. · -- If `u < m ^^^ n`, then either `u ^^^ n < m` or `u ^^^ m < n`. obtain ⟨u, rfl⟩ := Ordinal.lt_omega.1 (hu.trans (Ordinal.nat_lt_omega _)) replace hu := Ordinal.nat_cast_lt.1 hu cases' Nat.lt_xor_cases hu with h h -- In the first case, reducing the `m` pile to `u ^^^ n` gives the desired Grundy value. · refine' ⟨toLeftMovesAdd (Sum.inl <| toLeftMovesNim ⟨_, Ordinal.nat_cast_lt.2 h⟩), _⟩ simp [Nat.lxor_cancel_right, hn _ h] -- In the second case, reducing the `n` pile to `u ^^^ m` gives the desired Grundy value. · refine' ⟨toLeftMovesAdd (Sum.inr <| toLeftMovesNim ⟨_, Ordinal.nat_cast_lt.2 h⟩), _⟩ have : n ^^^ (u ^^^ n) = u; rw [Nat.xor_comm u, Nat.xor_cancel_left] simpa [hm _ h] using this #align pgame.grundy_value_nim_add_nim SetTheory.PGame.grundyValue_nim_add_nim theorem nim_add_nim_equiv {n m : ℕ} : nim n + nim m ≈ nim (n ^^^ m) := by rw [← grundyValue_eq_iff_equiv_nim, grundyValue_nim_add_nim] #align pgame.nim_add_nim_equiv SetTheory.PGame.nim_add_nim_equiv theorem grundyValue_add (G H : PGame) [G.Impartial] [H.Impartial] {n m : ℕ} (hG : grundyValue G = n) (hH : grundyValue H = m) : grundyValue (G + H) = n ^^^ m := by rw [← nim_grundyValue (n ^^^ m), grundyValue_eq_iff_equiv] refine' Equiv.trans _ nim_add_nim_equiv convert add_congr (equiv_nim_grundyValue G) (equiv_nim_grundyValue H) <;>
simp only [hG, hH]
theorem grundyValue_add (G H : PGame) [G.Impartial] [H.Impartial] {n m : ℕ} (hG : grundyValue G = n) (hH : grundyValue H = m) : grundyValue (G + H) = n ^^^ m := by rw [← nim_grundyValue (n ^^^ m), grundyValue_eq_iff_equiv] refine' Equiv.trans _ nim_add_nim_equiv convert add_congr (equiv_nim_grundyValue G) (equiv_nim_grundyValue H) <;>
Mathlib.SetTheory.Game.Nim.406_0.mmFMhRYSjViKjcP
theorem grundyValue_add (G H : PGame) [G.Impartial] [H.Impartial] {n m : ℕ} (hG : grundyValue G = n) (hH : grundyValue H = m) : grundyValue (G + H) = n ^^^ m
Mathlib_SetTheory_Game_Nim
β : Type v f : β → Type v P : Type v s : (b : β) → P ⟶ f b b : β x : P ⊢ Pi.π f b (Pi.lift s x) = s b x
/- Copyright (c) 2020 Scott Morrison. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Scott Morrison -/ import Mathlib.CategoryTheory.Limits.Types import Mathlib.CategoryTheory.Limits.Shapes.Products import Mathlib.CategoryTheory.Limits.Shapes.BinaryProducts import Mathlib.CategoryTheory.Limits.Shapes.Terminal import Mathlib.CategoryTheory.ConcreteCategory.Basic import Mathlib.Tactic.CategoryTheory.Elementwise #align_import category_theory.limits.shapes.types from "leanprover-community/mathlib"@"5dc6092d09e5e489106865241986f7f2ad28d4c8" /-! # Special shapes for limits in `Type`. The general shape (co)limits defined in `CategoryTheory.Limits.Types` are intended for use through the limits API, and the actual implementation should mostly be considered "sealed". In this file, we provide definitions of the "standard" special shapes of limits in `Type`, giving the expected definitional implementation: * the terminal object is `PUnit` * the binary product of `X` and `Y` is `X × Y` * the product of a family `f : J → Type` is `Π j, f j` * the coproduct of a family `f : J → Type` is `Σ j, f j` * the binary coproduct of `X` and `Y` is the sum type `X ⊕ Y` * the equalizer of a pair of maps `(g, h)` is the subtype `{x : Y // g x = h x}` * the coequalizer of a pair of maps `(f, g)` is the quotient of `Y` by `∀ x : Y, f x ~ g x` * the pullback of `f : X ⟶ Z` and `g : Y ⟶ Z` is the subtype `{ p : X × Y // f p.1 = g p.2 }` of the product We first construct terms of `IsLimit` and `LimitCone`, and then provide isomorphisms with the types generated by the `HasLimit` API. As an example, when setting up the monoidal category structure on `Type` we use the `Types.terminalLimitCone` and `Types.binaryProductLimitCone` definitions. -/ universe v u open CategoryTheory Limits namespace CategoryTheory.Limits.Types example : HasProducts.{v} (Type v) := inferInstance example [UnivLE.{v, u}] : HasProducts.{v} (Type u) := inferInstance -- This shortcut instance is required in `Mathlib.CategoryTheory.Closed.Types`, -- although I don't understand why, and wish it wasn't. instance : HasProducts.{v} (Type v) := inferInstance /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`. -/ @[simp 1001] theorem pi_lift_π_apply {β : Type v} [Small.{u} β] (f : β → Type u) {P : Type u} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := congr_fun (limit.lift_π (Fan.mk P s) ⟨b⟩) x #align category_theory.limits.types.pi_lift_π_apply CategoryTheory.Limits.Types.pi_lift_π_apply /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`, with specialized universes. -/ theorem pi_lift_π_apply' {β : Type v} (f : β → Type v) {P : Type v} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := by
simp
/-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`, with specialized universes. -/ theorem pi_lift_π_apply' {β : Type v} (f : β → Type v) {P : Type v} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := by
Mathlib.CategoryTheory.Limits.Shapes.Types.63_0.ctQAUYXLRXnvMGw
/-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`, with specialized universes. -/ theorem pi_lift_π_apply' {β : Type v} (f : β → Type v) {P : Type v} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x
Mathlib_CategoryTheory_Limits_Shapes_Types
β : Type v f g : β → Type v α : (j : β) → f j ⟶ g j b : β x : ∏ fun b => f b ⊢ Pi.π g b (Pi.map α x) = α b (Pi.π f b x)
/- Copyright (c) 2020 Scott Morrison. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Scott Morrison -/ import Mathlib.CategoryTheory.Limits.Types import Mathlib.CategoryTheory.Limits.Shapes.Products import Mathlib.CategoryTheory.Limits.Shapes.BinaryProducts import Mathlib.CategoryTheory.Limits.Shapes.Terminal import Mathlib.CategoryTheory.ConcreteCategory.Basic import Mathlib.Tactic.CategoryTheory.Elementwise #align_import category_theory.limits.shapes.types from "leanprover-community/mathlib"@"5dc6092d09e5e489106865241986f7f2ad28d4c8" /-! # Special shapes for limits in `Type`. The general shape (co)limits defined in `CategoryTheory.Limits.Types` are intended for use through the limits API, and the actual implementation should mostly be considered "sealed". In this file, we provide definitions of the "standard" special shapes of limits in `Type`, giving the expected definitional implementation: * the terminal object is `PUnit` * the binary product of `X` and `Y` is `X × Y` * the product of a family `f : J → Type` is `Π j, f j` * the coproduct of a family `f : J → Type` is `Σ j, f j` * the binary coproduct of `X` and `Y` is the sum type `X ⊕ Y` * the equalizer of a pair of maps `(g, h)` is the subtype `{x : Y // g x = h x}` * the coequalizer of a pair of maps `(f, g)` is the quotient of `Y` by `∀ x : Y, f x ~ g x` * the pullback of `f : X ⟶ Z` and `g : Y ⟶ Z` is the subtype `{ p : X × Y // f p.1 = g p.2 }` of the product We first construct terms of `IsLimit` and `LimitCone`, and then provide isomorphisms with the types generated by the `HasLimit` API. As an example, when setting up the monoidal category structure on `Type` we use the `Types.terminalLimitCone` and `Types.binaryProductLimitCone` definitions. -/ universe v u open CategoryTheory Limits namespace CategoryTheory.Limits.Types example : HasProducts.{v} (Type v) := inferInstance example [UnivLE.{v, u}] : HasProducts.{v} (Type u) := inferInstance -- This shortcut instance is required in `Mathlib.CategoryTheory.Closed.Types`, -- although I don't understand why, and wish it wasn't. instance : HasProducts.{v} (Type v) := inferInstance /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`. -/ @[simp 1001] theorem pi_lift_π_apply {β : Type v} [Small.{u} β] (f : β → Type u) {P : Type u} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := congr_fun (limit.lift_π (Fan.mk P s) ⟨b⟩) x #align category_theory.limits.types.pi_lift_π_apply CategoryTheory.Limits.Types.pi_lift_π_apply /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`, with specialized universes. -/ theorem pi_lift_π_apply' {β : Type v} (f : β → Type v) {P : Type v} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := by simp #align category_theory.limits.types.pi_lift_π_apply' CategoryTheory.Limits.Types.pi_lift_π_apply' /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`. -/ @[simp 1001] theorem pi_map_π_apply {β : Type v} [Small.{u} β] {f g : β → Type u} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := Limit.map_π_apply.{v, u} _ _ _ #align category_theory.limits.types.pi_map_π_apply CategoryTheory.Limits.Types.pi_map_π_apply /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`, with specialized universes. -/ theorem pi_map_π_apply' {β : Type v} {f g : β → Type v} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := by
simp
/-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`, with specialized universes. -/ theorem pi_map_π_apply' {β : Type v} {f g : β → Type v} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := by
Mathlib.CategoryTheory.Limits.Shapes.Types.79_0.ctQAUYXLRXnvMGw
/-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`, with specialized universes. -/ theorem pi_map_π_apply' {β : Type v} {f g : β → Type v} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x)
Mathlib_CategoryTheory_Limits_Shapes_Types
x✝ : Cone (Functor.empty (Type u)) ⊢ ∀ (j : Discrete PEmpty.{?u.3735 + 1}), (fun x x => PUnit.unit) x✝ ≫ { pt := PUnit.{u + 1}, π := (Functor.uniqueFromEmpty ((Functor.const (Discrete PEmpty.{?u.3735 + 1})).obj PUnit.{u + 1})).hom }.π.app j = x✝.π.app j
/- Copyright (c) 2020 Scott Morrison. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Scott Morrison -/ import Mathlib.CategoryTheory.Limits.Types import Mathlib.CategoryTheory.Limits.Shapes.Products import Mathlib.CategoryTheory.Limits.Shapes.BinaryProducts import Mathlib.CategoryTheory.Limits.Shapes.Terminal import Mathlib.CategoryTheory.ConcreteCategory.Basic import Mathlib.Tactic.CategoryTheory.Elementwise #align_import category_theory.limits.shapes.types from "leanprover-community/mathlib"@"5dc6092d09e5e489106865241986f7f2ad28d4c8" /-! # Special shapes for limits in `Type`. The general shape (co)limits defined in `CategoryTheory.Limits.Types` are intended for use through the limits API, and the actual implementation should mostly be considered "sealed". In this file, we provide definitions of the "standard" special shapes of limits in `Type`, giving the expected definitional implementation: * the terminal object is `PUnit` * the binary product of `X` and `Y` is `X × Y` * the product of a family `f : J → Type` is `Π j, f j` * the coproduct of a family `f : J → Type` is `Σ j, f j` * the binary coproduct of `X` and `Y` is the sum type `X ⊕ Y` * the equalizer of a pair of maps `(g, h)` is the subtype `{x : Y // g x = h x}` * the coequalizer of a pair of maps `(f, g)` is the quotient of `Y` by `∀ x : Y, f x ~ g x` * the pullback of `f : X ⟶ Z` and `g : Y ⟶ Z` is the subtype `{ p : X × Y // f p.1 = g p.2 }` of the product We first construct terms of `IsLimit` and `LimitCone`, and then provide isomorphisms with the types generated by the `HasLimit` API. As an example, when setting up the monoidal category structure on `Type` we use the `Types.terminalLimitCone` and `Types.binaryProductLimitCone` definitions. -/ universe v u open CategoryTheory Limits namespace CategoryTheory.Limits.Types example : HasProducts.{v} (Type v) := inferInstance example [UnivLE.{v, u}] : HasProducts.{v} (Type u) := inferInstance -- This shortcut instance is required in `Mathlib.CategoryTheory.Closed.Types`, -- although I don't understand why, and wish it wasn't. instance : HasProducts.{v} (Type v) := inferInstance /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`. -/ @[simp 1001] theorem pi_lift_π_apply {β : Type v} [Small.{u} β] (f : β → Type u) {P : Type u} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := congr_fun (limit.lift_π (Fan.mk P s) ⟨b⟩) x #align category_theory.limits.types.pi_lift_π_apply CategoryTheory.Limits.Types.pi_lift_π_apply /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`, with specialized universes. -/ theorem pi_lift_π_apply' {β : Type v} (f : β → Type v) {P : Type v} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := by simp #align category_theory.limits.types.pi_lift_π_apply' CategoryTheory.Limits.Types.pi_lift_π_apply' /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`. -/ @[simp 1001] theorem pi_map_π_apply {β : Type v} [Small.{u} β] {f g : β → Type u} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := Limit.map_π_apply.{v, u} _ _ _ #align category_theory.limits.types.pi_map_π_apply CategoryTheory.Limits.Types.pi_map_π_apply /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`, with specialized universes. -/ theorem pi_map_π_apply' {β : Type v} {f g : β → Type v} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := by simp #align category_theory.limits.types.pi_map_π_apply' CategoryTheory.Limits.Types.pi_map_π_apply' /-- The category of types has `PUnit` as a terminal object. -/ def terminalLimitCone : Limits.LimitCone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cone := { pt := PUnit π := (Functor.uniqueFromEmpty _).hom } isLimit := { lift := fun _ _ => PUnit.unit fac := fun _ => by
rintro ⟨⟨⟩⟩
/-- The category of types has `PUnit` as a terminal object. -/ def terminalLimitCone : Limits.LimitCone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cone := { pt := PUnit π := (Functor.uniqueFromEmpty _).hom } isLimit := { lift := fun _ _ => PUnit.unit fac := fun _ => by
Mathlib.CategoryTheory.Limits.Shapes.Types.86_0.ctQAUYXLRXnvMGw
/-- The category of types has `PUnit` as a terminal object. -/ def terminalLimitCone : Limits.LimitCone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cone
Mathlib_CategoryTheory_Limits_Shapes_Types
x✝² : Cone (Functor.empty (Type u)) x✝¹ : x✝².pt ⟶ { pt := PUnit.{u + 1}, π := (Functor.uniqueFromEmpty ((Functor.const (Discrete PEmpty.{?u.3735 + 1})).obj PUnit.{u + 1})).hom }.pt x✝ : ∀ (j : Discrete PEmpty.{?u.3735 + 1}), x✝¹ ≫ { pt := PUnit.{u + 1}, π := (Functor.uniqueFromEmpty ((Functor.const (Discrete PEmpty.{?u.3735 + 1})).obj PUnit.{u + 1})).hom }.π.app j = x✝².π.app j ⊢ x✝¹ = (fun x x => PUnit.unit) x✝²
/- Copyright (c) 2020 Scott Morrison. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Scott Morrison -/ import Mathlib.CategoryTheory.Limits.Types import Mathlib.CategoryTheory.Limits.Shapes.Products import Mathlib.CategoryTheory.Limits.Shapes.BinaryProducts import Mathlib.CategoryTheory.Limits.Shapes.Terminal import Mathlib.CategoryTheory.ConcreteCategory.Basic import Mathlib.Tactic.CategoryTheory.Elementwise #align_import category_theory.limits.shapes.types from "leanprover-community/mathlib"@"5dc6092d09e5e489106865241986f7f2ad28d4c8" /-! # Special shapes for limits in `Type`. The general shape (co)limits defined in `CategoryTheory.Limits.Types` are intended for use through the limits API, and the actual implementation should mostly be considered "sealed". In this file, we provide definitions of the "standard" special shapes of limits in `Type`, giving the expected definitional implementation: * the terminal object is `PUnit` * the binary product of `X` and `Y` is `X × Y` * the product of a family `f : J → Type` is `Π j, f j` * the coproduct of a family `f : J → Type` is `Σ j, f j` * the binary coproduct of `X` and `Y` is the sum type `X ⊕ Y` * the equalizer of a pair of maps `(g, h)` is the subtype `{x : Y // g x = h x}` * the coequalizer of a pair of maps `(f, g)` is the quotient of `Y` by `∀ x : Y, f x ~ g x` * the pullback of `f : X ⟶ Z` and `g : Y ⟶ Z` is the subtype `{ p : X × Y // f p.1 = g p.2 }` of the product We first construct terms of `IsLimit` and `LimitCone`, and then provide isomorphisms with the types generated by the `HasLimit` API. As an example, when setting up the monoidal category structure on `Type` we use the `Types.terminalLimitCone` and `Types.binaryProductLimitCone` definitions. -/ universe v u open CategoryTheory Limits namespace CategoryTheory.Limits.Types example : HasProducts.{v} (Type v) := inferInstance example [UnivLE.{v, u}] : HasProducts.{v} (Type u) := inferInstance -- This shortcut instance is required in `Mathlib.CategoryTheory.Closed.Types`, -- although I don't understand why, and wish it wasn't. instance : HasProducts.{v} (Type v) := inferInstance /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`. -/ @[simp 1001] theorem pi_lift_π_apply {β : Type v} [Small.{u} β] (f : β → Type u) {P : Type u} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := congr_fun (limit.lift_π (Fan.mk P s) ⟨b⟩) x #align category_theory.limits.types.pi_lift_π_apply CategoryTheory.Limits.Types.pi_lift_π_apply /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`, with specialized universes. -/ theorem pi_lift_π_apply' {β : Type v} (f : β → Type v) {P : Type v} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := by simp #align category_theory.limits.types.pi_lift_π_apply' CategoryTheory.Limits.Types.pi_lift_π_apply' /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`. -/ @[simp 1001] theorem pi_map_π_apply {β : Type v} [Small.{u} β] {f g : β → Type u} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := Limit.map_π_apply.{v, u} _ _ _ #align category_theory.limits.types.pi_map_π_apply CategoryTheory.Limits.Types.pi_map_π_apply /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`, with specialized universes. -/ theorem pi_map_π_apply' {β : Type v} {f g : β → Type v} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := by simp #align category_theory.limits.types.pi_map_π_apply' CategoryTheory.Limits.Types.pi_map_π_apply' /-- The category of types has `PUnit` as a terminal object. -/ def terminalLimitCone : Limits.LimitCone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cone := { pt := PUnit π := (Functor.uniqueFromEmpty _).hom } isLimit := { lift := fun _ _ => PUnit.unit fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by
funext
/-- The category of types has `PUnit` as a terminal object. -/ def terminalLimitCone : Limits.LimitCone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cone := { pt := PUnit π := (Functor.uniqueFromEmpty _).hom } isLimit := { lift := fun _ _ => PUnit.unit fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by
Mathlib.CategoryTheory.Limits.Shapes.Types.86_0.ctQAUYXLRXnvMGw
/-- The category of types has `PUnit` as a terminal object. -/ def terminalLimitCone : Limits.LimitCone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cone
Mathlib_CategoryTheory_Limits_Shapes_Types
case h x✝³ : Cone (Functor.empty (Type u)) x✝² : x✝³.pt ⟶ { pt := PUnit.{u + 1}, π := (Functor.uniqueFromEmpty ((Functor.const (Discrete PEmpty.{?u.3735 + 1})).obj PUnit.{u + 1})).hom }.pt x✝¹ : ∀ (j : Discrete PEmpty.{?u.3735 + 1}), x✝² ≫ { pt := PUnit.{u + 1}, π := (Functor.uniqueFromEmpty ((Functor.const (Discrete PEmpty.{?u.3735 + 1})).obj PUnit.{u + 1})).hom }.π.app j = x✝³.π.app j x✝ : x✝³.pt ⊢ x✝² x✝ = (fun x x => PUnit.unit) x✝³ x✝
/- Copyright (c) 2020 Scott Morrison. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Scott Morrison -/ import Mathlib.CategoryTheory.Limits.Types import Mathlib.CategoryTheory.Limits.Shapes.Products import Mathlib.CategoryTheory.Limits.Shapes.BinaryProducts import Mathlib.CategoryTheory.Limits.Shapes.Terminal import Mathlib.CategoryTheory.ConcreteCategory.Basic import Mathlib.Tactic.CategoryTheory.Elementwise #align_import category_theory.limits.shapes.types from "leanprover-community/mathlib"@"5dc6092d09e5e489106865241986f7f2ad28d4c8" /-! # Special shapes for limits in `Type`. The general shape (co)limits defined in `CategoryTheory.Limits.Types` are intended for use through the limits API, and the actual implementation should mostly be considered "sealed". In this file, we provide definitions of the "standard" special shapes of limits in `Type`, giving the expected definitional implementation: * the terminal object is `PUnit` * the binary product of `X` and `Y` is `X × Y` * the product of a family `f : J → Type` is `Π j, f j` * the coproduct of a family `f : J → Type` is `Σ j, f j` * the binary coproduct of `X` and `Y` is the sum type `X ⊕ Y` * the equalizer of a pair of maps `(g, h)` is the subtype `{x : Y // g x = h x}` * the coequalizer of a pair of maps `(f, g)` is the quotient of `Y` by `∀ x : Y, f x ~ g x` * the pullback of `f : X ⟶ Z` and `g : Y ⟶ Z` is the subtype `{ p : X × Y // f p.1 = g p.2 }` of the product We first construct terms of `IsLimit` and `LimitCone`, and then provide isomorphisms with the types generated by the `HasLimit` API. As an example, when setting up the monoidal category structure on `Type` we use the `Types.terminalLimitCone` and `Types.binaryProductLimitCone` definitions. -/ universe v u open CategoryTheory Limits namespace CategoryTheory.Limits.Types example : HasProducts.{v} (Type v) := inferInstance example [UnivLE.{v, u}] : HasProducts.{v} (Type u) := inferInstance -- This shortcut instance is required in `Mathlib.CategoryTheory.Closed.Types`, -- although I don't understand why, and wish it wasn't. instance : HasProducts.{v} (Type v) := inferInstance /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`. -/ @[simp 1001] theorem pi_lift_π_apply {β : Type v} [Small.{u} β] (f : β → Type u) {P : Type u} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := congr_fun (limit.lift_π (Fan.mk P s) ⟨b⟩) x #align category_theory.limits.types.pi_lift_π_apply CategoryTheory.Limits.Types.pi_lift_π_apply /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`, with specialized universes. -/ theorem pi_lift_π_apply' {β : Type v} (f : β → Type v) {P : Type v} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := by simp #align category_theory.limits.types.pi_lift_π_apply' CategoryTheory.Limits.Types.pi_lift_π_apply' /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`. -/ @[simp 1001] theorem pi_map_π_apply {β : Type v} [Small.{u} β] {f g : β → Type u} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := Limit.map_π_apply.{v, u} _ _ _ #align category_theory.limits.types.pi_map_π_apply CategoryTheory.Limits.Types.pi_map_π_apply /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`, with specialized universes. -/ theorem pi_map_π_apply' {β : Type v} {f g : β → Type v} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := by simp #align category_theory.limits.types.pi_map_π_apply' CategoryTheory.Limits.Types.pi_map_π_apply' /-- The category of types has `PUnit` as a terminal object. -/ def terminalLimitCone : Limits.LimitCone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cone := { pt := PUnit π := (Functor.uniqueFromEmpty _).hom } isLimit := { lift := fun _ _ => PUnit.unit fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext
apply Subsingleton.elim
/-- The category of types has `PUnit` as a terminal object. -/ def terminalLimitCone : Limits.LimitCone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cone := { pt := PUnit π := (Functor.uniqueFromEmpty _).hom } isLimit := { lift := fun _ _ => PUnit.unit fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext
Mathlib.CategoryTheory.Limits.Shapes.Types.86_0.ctQAUYXLRXnvMGw
/-- The category of types has `PUnit` as a terminal object. -/ def terminalLimitCone : Limits.LimitCone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cone
Mathlib_CategoryTheory_Limits_Shapes_Types
X : Type u ⊢ IsTerminal X ≃ (X ≅ PUnit.{u + 1})
/- Copyright (c) 2020 Scott Morrison. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Scott Morrison -/ import Mathlib.CategoryTheory.Limits.Types import Mathlib.CategoryTheory.Limits.Shapes.Products import Mathlib.CategoryTheory.Limits.Shapes.BinaryProducts import Mathlib.CategoryTheory.Limits.Shapes.Terminal import Mathlib.CategoryTheory.ConcreteCategory.Basic import Mathlib.Tactic.CategoryTheory.Elementwise #align_import category_theory.limits.shapes.types from "leanprover-community/mathlib"@"5dc6092d09e5e489106865241986f7f2ad28d4c8" /-! # Special shapes for limits in `Type`. The general shape (co)limits defined in `CategoryTheory.Limits.Types` are intended for use through the limits API, and the actual implementation should mostly be considered "sealed". In this file, we provide definitions of the "standard" special shapes of limits in `Type`, giving the expected definitional implementation: * the terminal object is `PUnit` * the binary product of `X` and `Y` is `X × Y` * the product of a family `f : J → Type` is `Π j, f j` * the coproduct of a family `f : J → Type` is `Σ j, f j` * the binary coproduct of `X` and `Y` is the sum type `X ⊕ Y` * the equalizer of a pair of maps `(g, h)` is the subtype `{x : Y // g x = h x}` * the coequalizer of a pair of maps `(f, g)` is the quotient of `Y` by `∀ x : Y, f x ~ g x` * the pullback of `f : X ⟶ Z` and `g : Y ⟶ Z` is the subtype `{ p : X × Y // f p.1 = g p.2 }` of the product We first construct terms of `IsLimit` and `LimitCone`, and then provide isomorphisms with the types generated by the `HasLimit` API. As an example, when setting up the monoidal category structure on `Type` we use the `Types.terminalLimitCone` and `Types.binaryProductLimitCone` definitions. -/ universe v u open CategoryTheory Limits namespace CategoryTheory.Limits.Types example : HasProducts.{v} (Type v) := inferInstance example [UnivLE.{v, u}] : HasProducts.{v} (Type u) := inferInstance -- This shortcut instance is required in `Mathlib.CategoryTheory.Closed.Types`, -- although I don't understand why, and wish it wasn't. instance : HasProducts.{v} (Type v) := inferInstance /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`. -/ @[simp 1001] theorem pi_lift_π_apply {β : Type v} [Small.{u} β] (f : β → Type u) {P : Type u} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := congr_fun (limit.lift_π (Fan.mk P s) ⟨b⟩) x #align category_theory.limits.types.pi_lift_π_apply CategoryTheory.Limits.Types.pi_lift_π_apply /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`, with specialized universes. -/ theorem pi_lift_π_apply' {β : Type v} (f : β → Type v) {P : Type v} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := by simp #align category_theory.limits.types.pi_lift_π_apply' CategoryTheory.Limits.Types.pi_lift_π_apply' /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`. -/ @[simp 1001] theorem pi_map_π_apply {β : Type v} [Small.{u} β] {f g : β → Type u} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := Limit.map_π_apply.{v, u} _ _ _ #align category_theory.limits.types.pi_map_π_apply CategoryTheory.Limits.Types.pi_map_π_apply /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`, with specialized universes. -/ theorem pi_map_π_apply' {β : Type v} {f g : β → Type v} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := by simp #align category_theory.limits.types.pi_map_π_apply' CategoryTheory.Limits.Types.pi_map_π_apply' /-- The category of types has `PUnit` as a terminal object. -/ def terminalLimitCone : Limits.LimitCone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cone := { pt := PUnit π := (Functor.uniqueFromEmpty _).hom } isLimit := { lift := fun _ _ => PUnit.unit fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext apply Subsingleton.elim } #align category_theory.limits.types.terminal_limit_cone CategoryTheory.Limits.Types.terminalLimitCone /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def terminalIso : ⊤_ Type u ≅ PUnit := limit.isoLimitCone terminalLimitCone.{u, 0} #align category_theory.limits.types.terminal_iso CategoryTheory.Limits.Types.terminalIso /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def isTerminalPunit : IsTerminal (PUnit : Type u) := terminalIsTerminal.ofIso terminalIso #align category_theory.limits.types.is_terminal_punit CategoryTheory.Limits.Types.isTerminalPunit -- porting note: the following three instances have been added to ease -- the automation in a definition in `AlgebraicTopology.SimplicialSet` noncomputable instance : Inhabited (⊤_ (Type u)) := ⟨@terminal.from (Type u) _ _ (ULift (Fin 1)) (ULift.up 0)⟩ instance : Subsingleton (⊤_ (Type u)) := ⟨fun a b => congr_fun (@Subsingleton.elim (_ ⟶ ⊤_ (Type u)) _ (fun _ => a) (fun _ => b)) (ULift.up (0 : Fin 1))⟩ noncomputable instance : Unique (⊤_ (Type u)) := Unique.mk' _ /-- A type is terminal if and only if it contains exactly one element. -/ noncomputable def isTerminalEquivUnique (X : Type u) : IsTerminal X ≃ Unique X := equivOfSubsingletonOfSubsingleton (fun h => ((Iso.toEquiv (terminalIsoIsTerminal h).symm).unique)) (fun _ => IsTerminal.ofIso terminalIsTerminal (Equiv.toIso (Equiv.equivOfUnique _ _))) /-- A type is terminal if and only if it is isomorphic to `PUnit`. -/ noncomputable def isTerminalEquivIsoPUnit (X : Type u) : IsTerminal X ≃ (X ≅ PUnit) := by
calc IsTerminal X ≃ Unique X := isTerminalEquivUnique _ _ ≃ (X ≃ PUnit.{u + 1}) := uniqueEquivEquivUnique _ _ _ ≃ (X ≅ PUnit) := equivEquivIso
/-- A type is terminal if and only if it is isomorphic to `PUnit`. -/ noncomputable def isTerminalEquivIsoPUnit (X : Type u) : IsTerminal X ≃ (X ≅ PUnit) := by
Mathlib.CategoryTheory.Limits.Shapes.Types.127_0.ctQAUYXLRXnvMGw
/-- A type is terminal if and only if it is isomorphic to `PUnit`. -/ noncomputable def isTerminalEquivIsoPUnit (X : Type u) : IsTerminal X ≃ (X ≅ PUnit)
Mathlib_CategoryTheory_Limits_Shapes_Types
x✝ : Cocone (Functor.empty (Type u)) ⊢ { pt := PEmpty.{u + 1}, ι := (Functor.uniqueFromEmpty ((Functor.const (Discrete PEmpty.{?u.11885 + 1})).obj PEmpty.{u + 1})).inv }.pt ⟶ x✝.pt
/- Copyright (c) 2020 Scott Morrison. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Scott Morrison -/ import Mathlib.CategoryTheory.Limits.Types import Mathlib.CategoryTheory.Limits.Shapes.Products import Mathlib.CategoryTheory.Limits.Shapes.BinaryProducts import Mathlib.CategoryTheory.Limits.Shapes.Terminal import Mathlib.CategoryTheory.ConcreteCategory.Basic import Mathlib.Tactic.CategoryTheory.Elementwise #align_import category_theory.limits.shapes.types from "leanprover-community/mathlib"@"5dc6092d09e5e489106865241986f7f2ad28d4c8" /-! # Special shapes for limits in `Type`. The general shape (co)limits defined in `CategoryTheory.Limits.Types` are intended for use through the limits API, and the actual implementation should mostly be considered "sealed". In this file, we provide definitions of the "standard" special shapes of limits in `Type`, giving the expected definitional implementation: * the terminal object is `PUnit` * the binary product of `X` and `Y` is `X × Y` * the product of a family `f : J → Type` is `Π j, f j` * the coproduct of a family `f : J → Type` is `Σ j, f j` * the binary coproduct of `X` and `Y` is the sum type `X ⊕ Y` * the equalizer of a pair of maps `(g, h)` is the subtype `{x : Y // g x = h x}` * the coequalizer of a pair of maps `(f, g)` is the quotient of `Y` by `∀ x : Y, f x ~ g x` * the pullback of `f : X ⟶ Z` and `g : Y ⟶ Z` is the subtype `{ p : X × Y // f p.1 = g p.2 }` of the product We first construct terms of `IsLimit` and `LimitCone`, and then provide isomorphisms with the types generated by the `HasLimit` API. As an example, when setting up the monoidal category structure on `Type` we use the `Types.terminalLimitCone` and `Types.binaryProductLimitCone` definitions. -/ universe v u open CategoryTheory Limits namespace CategoryTheory.Limits.Types example : HasProducts.{v} (Type v) := inferInstance example [UnivLE.{v, u}] : HasProducts.{v} (Type u) := inferInstance -- This shortcut instance is required in `Mathlib.CategoryTheory.Closed.Types`, -- although I don't understand why, and wish it wasn't. instance : HasProducts.{v} (Type v) := inferInstance /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`. -/ @[simp 1001] theorem pi_lift_π_apply {β : Type v} [Small.{u} β] (f : β → Type u) {P : Type u} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := congr_fun (limit.lift_π (Fan.mk P s) ⟨b⟩) x #align category_theory.limits.types.pi_lift_π_apply CategoryTheory.Limits.Types.pi_lift_π_apply /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`, with specialized universes. -/ theorem pi_lift_π_apply' {β : Type v} (f : β → Type v) {P : Type v} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := by simp #align category_theory.limits.types.pi_lift_π_apply' CategoryTheory.Limits.Types.pi_lift_π_apply' /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`. -/ @[simp 1001] theorem pi_map_π_apply {β : Type v} [Small.{u} β] {f g : β → Type u} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := Limit.map_π_apply.{v, u} _ _ _ #align category_theory.limits.types.pi_map_π_apply CategoryTheory.Limits.Types.pi_map_π_apply /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`, with specialized universes. -/ theorem pi_map_π_apply' {β : Type v} {f g : β → Type v} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := by simp #align category_theory.limits.types.pi_map_π_apply' CategoryTheory.Limits.Types.pi_map_π_apply' /-- The category of types has `PUnit` as a terminal object. -/ def terminalLimitCone : Limits.LimitCone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cone := { pt := PUnit π := (Functor.uniqueFromEmpty _).hom } isLimit := { lift := fun _ _ => PUnit.unit fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext apply Subsingleton.elim } #align category_theory.limits.types.terminal_limit_cone CategoryTheory.Limits.Types.terminalLimitCone /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def terminalIso : ⊤_ Type u ≅ PUnit := limit.isoLimitCone terminalLimitCone.{u, 0} #align category_theory.limits.types.terminal_iso CategoryTheory.Limits.Types.terminalIso /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def isTerminalPunit : IsTerminal (PUnit : Type u) := terminalIsTerminal.ofIso terminalIso #align category_theory.limits.types.is_terminal_punit CategoryTheory.Limits.Types.isTerminalPunit -- porting note: the following three instances have been added to ease -- the automation in a definition in `AlgebraicTopology.SimplicialSet` noncomputable instance : Inhabited (⊤_ (Type u)) := ⟨@terminal.from (Type u) _ _ (ULift (Fin 1)) (ULift.up 0)⟩ instance : Subsingleton (⊤_ (Type u)) := ⟨fun a b => congr_fun (@Subsingleton.elim (_ ⟶ ⊤_ (Type u)) _ (fun _ => a) (fun _ => b)) (ULift.up (0 : Fin 1))⟩ noncomputable instance : Unique (⊤_ (Type u)) := Unique.mk' _ /-- A type is terminal if and only if it contains exactly one element. -/ noncomputable def isTerminalEquivUnique (X : Type u) : IsTerminal X ≃ Unique X := equivOfSubsingletonOfSubsingleton (fun h => ((Iso.toEquiv (terminalIsoIsTerminal h).symm).unique)) (fun _ => IsTerminal.ofIso terminalIsTerminal (Equiv.toIso (Equiv.equivOfUnique _ _))) /-- A type is terminal if and only if it is isomorphic to `PUnit`. -/ noncomputable def isTerminalEquivIsoPUnit (X : Type u) : IsTerminal X ≃ (X ≅ PUnit) := by calc IsTerminal X ≃ Unique X := isTerminalEquivUnique _ _ ≃ (X ≃ PUnit.{u + 1}) := uniqueEquivEquivUnique _ _ _ ≃ (X ≅ PUnit) := equivEquivIso /-- The category of types has `PEmpty` as an initial object. -/ def initialColimitCocone : Limits.ColimitCocone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cocone := { pt := PEmpty ι := (Functor.uniqueFromEmpty _).inv } isColimit := { desc := fun _ => by
rintro ⟨⟩
/-- The category of types has `PEmpty` as an initial object. -/ def initialColimitCocone : Limits.ColimitCocone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cocone := { pt := PEmpty ι := (Functor.uniqueFromEmpty _).inv } isColimit := { desc := fun _ => by
Mathlib.CategoryTheory.Limits.Shapes.Types.134_0.ctQAUYXLRXnvMGw
/-- The category of types has `PEmpty` as an initial object. -/ def initialColimitCocone : Limits.ColimitCocone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cocone
Mathlib_CategoryTheory_Limits_Shapes_Types
x✝ : Cocone (Functor.empty (Type u)) ⊢ ∀ (j : Discrete PEmpty.{?u.11885 + 1}), { pt := PEmpty.{u + 1}, ι := (Functor.uniqueFromEmpty ((Functor.const (Discrete PEmpty.{?u.11885 + 1})).obj PEmpty.{u + 1})).inv }.ι.app j ≫ (fun x a => PEmpty.casesOn (fun x_1 => x.pt) a) x✝ = x✝.ι.app j
/- Copyright (c) 2020 Scott Morrison. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Scott Morrison -/ import Mathlib.CategoryTheory.Limits.Types import Mathlib.CategoryTheory.Limits.Shapes.Products import Mathlib.CategoryTheory.Limits.Shapes.BinaryProducts import Mathlib.CategoryTheory.Limits.Shapes.Terminal import Mathlib.CategoryTheory.ConcreteCategory.Basic import Mathlib.Tactic.CategoryTheory.Elementwise #align_import category_theory.limits.shapes.types from "leanprover-community/mathlib"@"5dc6092d09e5e489106865241986f7f2ad28d4c8" /-! # Special shapes for limits in `Type`. The general shape (co)limits defined in `CategoryTheory.Limits.Types` are intended for use through the limits API, and the actual implementation should mostly be considered "sealed". In this file, we provide definitions of the "standard" special shapes of limits in `Type`, giving the expected definitional implementation: * the terminal object is `PUnit` * the binary product of `X` and `Y` is `X × Y` * the product of a family `f : J → Type` is `Π j, f j` * the coproduct of a family `f : J → Type` is `Σ j, f j` * the binary coproduct of `X` and `Y` is the sum type `X ⊕ Y` * the equalizer of a pair of maps `(g, h)` is the subtype `{x : Y // g x = h x}` * the coequalizer of a pair of maps `(f, g)` is the quotient of `Y` by `∀ x : Y, f x ~ g x` * the pullback of `f : X ⟶ Z` and `g : Y ⟶ Z` is the subtype `{ p : X × Y // f p.1 = g p.2 }` of the product We first construct terms of `IsLimit` and `LimitCone`, and then provide isomorphisms with the types generated by the `HasLimit` API. As an example, when setting up the monoidal category structure on `Type` we use the `Types.terminalLimitCone` and `Types.binaryProductLimitCone` definitions. -/ universe v u open CategoryTheory Limits namespace CategoryTheory.Limits.Types example : HasProducts.{v} (Type v) := inferInstance example [UnivLE.{v, u}] : HasProducts.{v} (Type u) := inferInstance -- This shortcut instance is required in `Mathlib.CategoryTheory.Closed.Types`, -- although I don't understand why, and wish it wasn't. instance : HasProducts.{v} (Type v) := inferInstance /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`. -/ @[simp 1001] theorem pi_lift_π_apply {β : Type v} [Small.{u} β] (f : β → Type u) {P : Type u} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := congr_fun (limit.lift_π (Fan.mk P s) ⟨b⟩) x #align category_theory.limits.types.pi_lift_π_apply CategoryTheory.Limits.Types.pi_lift_π_apply /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`, with specialized universes. -/ theorem pi_lift_π_apply' {β : Type v} (f : β → Type v) {P : Type v} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := by simp #align category_theory.limits.types.pi_lift_π_apply' CategoryTheory.Limits.Types.pi_lift_π_apply' /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`. -/ @[simp 1001] theorem pi_map_π_apply {β : Type v} [Small.{u} β] {f g : β → Type u} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := Limit.map_π_apply.{v, u} _ _ _ #align category_theory.limits.types.pi_map_π_apply CategoryTheory.Limits.Types.pi_map_π_apply /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`, with specialized universes. -/ theorem pi_map_π_apply' {β : Type v} {f g : β → Type v} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := by simp #align category_theory.limits.types.pi_map_π_apply' CategoryTheory.Limits.Types.pi_map_π_apply' /-- The category of types has `PUnit` as a terminal object. -/ def terminalLimitCone : Limits.LimitCone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cone := { pt := PUnit π := (Functor.uniqueFromEmpty _).hom } isLimit := { lift := fun _ _ => PUnit.unit fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext apply Subsingleton.elim } #align category_theory.limits.types.terminal_limit_cone CategoryTheory.Limits.Types.terminalLimitCone /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def terminalIso : ⊤_ Type u ≅ PUnit := limit.isoLimitCone terminalLimitCone.{u, 0} #align category_theory.limits.types.terminal_iso CategoryTheory.Limits.Types.terminalIso /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def isTerminalPunit : IsTerminal (PUnit : Type u) := terminalIsTerminal.ofIso terminalIso #align category_theory.limits.types.is_terminal_punit CategoryTheory.Limits.Types.isTerminalPunit -- porting note: the following three instances have been added to ease -- the automation in a definition in `AlgebraicTopology.SimplicialSet` noncomputable instance : Inhabited (⊤_ (Type u)) := ⟨@terminal.from (Type u) _ _ (ULift (Fin 1)) (ULift.up 0)⟩ instance : Subsingleton (⊤_ (Type u)) := ⟨fun a b => congr_fun (@Subsingleton.elim (_ ⟶ ⊤_ (Type u)) _ (fun _ => a) (fun _ => b)) (ULift.up (0 : Fin 1))⟩ noncomputable instance : Unique (⊤_ (Type u)) := Unique.mk' _ /-- A type is terminal if and only if it contains exactly one element. -/ noncomputable def isTerminalEquivUnique (X : Type u) : IsTerminal X ≃ Unique X := equivOfSubsingletonOfSubsingleton (fun h => ((Iso.toEquiv (terminalIsoIsTerminal h).symm).unique)) (fun _ => IsTerminal.ofIso terminalIsTerminal (Equiv.toIso (Equiv.equivOfUnique _ _))) /-- A type is terminal if and only if it is isomorphic to `PUnit`. -/ noncomputable def isTerminalEquivIsoPUnit (X : Type u) : IsTerminal X ≃ (X ≅ PUnit) := by calc IsTerminal X ≃ Unique X := isTerminalEquivUnique _ _ ≃ (X ≃ PUnit.{u + 1}) := uniqueEquivEquivUnique _ _ _ ≃ (X ≅ PUnit) := equivEquivIso /-- The category of types has `PEmpty` as an initial object. -/ def initialColimitCocone : Limits.ColimitCocone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cocone := { pt := PEmpty ι := (Functor.uniqueFromEmpty _).inv } isColimit := { desc := fun _ => by rintro ⟨⟩ fac := fun _ => by
rintro ⟨⟨⟩⟩
/-- The category of types has `PEmpty` as an initial object. -/ def initialColimitCocone : Limits.ColimitCocone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cocone := { pt := PEmpty ι := (Functor.uniqueFromEmpty _).inv } isColimit := { desc := fun _ => by rintro ⟨⟩ fac := fun _ => by
Mathlib.CategoryTheory.Limits.Shapes.Types.134_0.ctQAUYXLRXnvMGw
/-- The category of types has `PEmpty` as an initial object. -/ def initialColimitCocone : Limits.ColimitCocone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cocone
Mathlib_CategoryTheory_Limits_Shapes_Types
x✝² : Cocone (Functor.empty (Type u)) x✝¹ : { pt := PEmpty.{u + 1}, ι := (Functor.uniqueFromEmpty ((Functor.const (Discrete PEmpty.{?u.11885 + 1})).obj PEmpty.{u + 1})).inv }.pt ⟶ x✝².pt x✝ : ∀ (j : Discrete PEmpty.{?u.11885 + 1}), { pt := PEmpty.{u + 1}, ι := (Functor.uniqueFromEmpty ((Functor.const (Discrete PEmpty.{?u.11885 + 1})).obj PEmpty.{u + 1})).inv }.ι.app j ≫ x✝¹ = x✝².ι.app j ⊢ x✝¹ = (fun x a => PEmpty.casesOn (fun x_1 => x.pt) a) x✝²
/- Copyright (c) 2020 Scott Morrison. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Scott Morrison -/ import Mathlib.CategoryTheory.Limits.Types import Mathlib.CategoryTheory.Limits.Shapes.Products import Mathlib.CategoryTheory.Limits.Shapes.BinaryProducts import Mathlib.CategoryTheory.Limits.Shapes.Terminal import Mathlib.CategoryTheory.ConcreteCategory.Basic import Mathlib.Tactic.CategoryTheory.Elementwise #align_import category_theory.limits.shapes.types from "leanprover-community/mathlib"@"5dc6092d09e5e489106865241986f7f2ad28d4c8" /-! # Special shapes for limits in `Type`. The general shape (co)limits defined in `CategoryTheory.Limits.Types` are intended for use through the limits API, and the actual implementation should mostly be considered "sealed". In this file, we provide definitions of the "standard" special shapes of limits in `Type`, giving the expected definitional implementation: * the terminal object is `PUnit` * the binary product of `X` and `Y` is `X × Y` * the product of a family `f : J → Type` is `Π j, f j` * the coproduct of a family `f : J → Type` is `Σ j, f j` * the binary coproduct of `X` and `Y` is the sum type `X ⊕ Y` * the equalizer of a pair of maps `(g, h)` is the subtype `{x : Y // g x = h x}` * the coequalizer of a pair of maps `(f, g)` is the quotient of `Y` by `∀ x : Y, f x ~ g x` * the pullback of `f : X ⟶ Z` and `g : Y ⟶ Z` is the subtype `{ p : X × Y // f p.1 = g p.2 }` of the product We first construct terms of `IsLimit` and `LimitCone`, and then provide isomorphisms with the types generated by the `HasLimit` API. As an example, when setting up the monoidal category structure on `Type` we use the `Types.terminalLimitCone` and `Types.binaryProductLimitCone` definitions. -/ universe v u open CategoryTheory Limits namespace CategoryTheory.Limits.Types example : HasProducts.{v} (Type v) := inferInstance example [UnivLE.{v, u}] : HasProducts.{v} (Type u) := inferInstance -- This shortcut instance is required in `Mathlib.CategoryTheory.Closed.Types`, -- although I don't understand why, and wish it wasn't. instance : HasProducts.{v} (Type v) := inferInstance /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`. -/ @[simp 1001] theorem pi_lift_π_apply {β : Type v} [Small.{u} β] (f : β → Type u) {P : Type u} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := congr_fun (limit.lift_π (Fan.mk P s) ⟨b⟩) x #align category_theory.limits.types.pi_lift_π_apply CategoryTheory.Limits.Types.pi_lift_π_apply /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`, with specialized universes. -/ theorem pi_lift_π_apply' {β : Type v} (f : β → Type v) {P : Type v} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := by simp #align category_theory.limits.types.pi_lift_π_apply' CategoryTheory.Limits.Types.pi_lift_π_apply' /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`. -/ @[simp 1001] theorem pi_map_π_apply {β : Type v} [Small.{u} β] {f g : β → Type u} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := Limit.map_π_apply.{v, u} _ _ _ #align category_theory.limits.types.pi_map_π_apply CategoryTheory.Limits.Types.pi_map_π_apply /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`, with specialized universes. -/ theorem pi_map_π_apply' {β : Type v} {f g : β → Type v} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := by simp #align category_theory.limits.types.pi_map_π_apply' CategoryTheory.Limits.Types.pi_map_π_apply' /-- The category of types has `PUnit` as a terminal object. -/ def terminalLimitCone : Limits.LimitCone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cone := { pt := PUnit π := (Functor.uniqueFromEmpty _).hom } isLimit := { lift := fun _ _ => PUnit.unit fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext apply Subsingleton.elim } #align category_theory.limits.types.terminal_limit_cone CategoryTheory.Limits.Types.terminalLimitCone /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def terminalIso : ⊤_ Type u ≅ PUnit := limit.isoLimitCone terminalLimitCone.{u, 0} #align category_theory.limits.types.terminal_iso CategoryTheory.Limits.Types.terminalIso /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def isTerminalPunit : IsTerminal (PUnit : Type u) := terminalIsTerminal.ofIso terminalIso #align category_theory.limits.types.is_terminal_punit CategoryTheory.Limits.Types.isTerminalPunit -- porting note: the following three instances have been added to ease -- the automation in a definition in `AlgebraicTopology.SimplicialSet` noncomputable instance : Inhabited (⊤_ (Type u)) := ⟨@terminal.from (Type u) _ _ (ULift (Fin 1)) (ULift.up 0)⟩ instance : Subsingleton (⊤_ (Type u)) := ⟨fun a b => congr_fun (@Subsingleton.elim (_ ⟶ ⊤_ (Type u)) _ (fun _ => a) (fun _ => b)) (ULift.up (0 : Fin 1))⟩ noncomputable instance : Unique (⊤_ (Type u)) := Unique.mk' _ /-- A type is terminal if and only if it contains exactly one element. -/ noncomputable def isTerminalEquivUnique (X : Type u) : IsTerminal X ≃ Unique X := equivOfSubsingletonOfSubsingleton (fun h => ((Iso.toEquiv (terminalIsoIsTerminal h).symm).unique)) (fun _ => IsTerminal.ofIso terminalIsTerminal (Equiv.toIso (Equiv.equivOfUnique _ _))) /-- A type is terminal if and only if it is isomorphic to `PUnit`. -/ noncomputable def isTerminalEquivIsoPUnit (X : Type u) : IsTerminal X ≃ (X ≅ PUnit) := by calc IsTerminal X ≃ Unique X := isTerminalEquivUnique _ _ ≃ (X ≃ PUnit.{u + 1}) := uniqueEquivEquivUnique _ _ _ ≃ (X ≅ PUnit) := equivEquivIso /-- The category of types has `PEmpty` as an initial object. -/ def initialColimitCocone : Limits.ColimitCocone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cocone := { pt := PEmpty ι := (Functor.uniqueFromEmpty _).inv } isColimit := { desc := fun _ => by rintro ⟨⟩ fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by
funext x
/-- The category of types has `PEmpty` as an initial object. -/ def initialColimitCocone : Limits.ColimitCocone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cocone := { pt := PEmpty ι := (Functor.uniqueFromEmpty _).inv } isColimit := { desc := fun _ => by rintro ⟨⟩ fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by
Mathlib.CategoryTheory.Limits.Shapes.Types.134_0.ctQAUYXLRXnvMGw
/-- The category of types has `PEmpty` as an initial object. -/ def initialColimitCocone : Limits.ColimitCocone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cocone
Mathlib_CategoryTheory_Limits_Shapes_Types
case h x✝² : Cocone (Functor.empty (Type u)) x✝¹ : { pt := PEmpty.{u + 1}, ι := (Functor.uniqueFromEmpty ((Functor.const (Discrete PEmpty.{?u.11885 + 1})).obj PEmpty.{u + 1})).inv }.pt ⟶ x✝².pt x✝ : ∀ (j : Discrete PEmpty.{?u.11885 + 1}), { pt := PEmpty.{u + 1}, ι := (Functor.uniqueFromEmpty ((Functor.const (Discrete PEmpty.{?u.11885 + 1})).obj PEmpty.{u + 1})).inv }.ι.app j ≫ x✝¹ = x✝².ι.app j x : { pt := PEmpty.{u + 1}, ι := (Functor.uniqueFromEmpty ((Functor.const (Discrete PEmpty.{?u.11885 + 1})).obj PEmpty.{u + 1})).inv }.pt ⊢ x✝¹ x = (fun x a => PEmpty.casesOn (fun x_1 => x.pt) a) x✝² x
/- Copyright (c) 2020 Scott Morrison. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Scott Morrison -/ import Mathlib.CategoryTheory.Limits.Types import Mathlib.CategoryTheory.Limits.Shapes.Products import Mathlib.CategoryTheory.Limits.Shapes.BinaryProducts import Mathlib.CategoryTheory.Limits.Shapes.Terminal import Mathlib.CategoryTheory.ConcreteCategory.Basic import Mathlib.Tactic.CategoryTheory.Elementwise #align_import category_theory.limits.shapes.types from "leanprover-community/mathlib"@"5dc6092d09e5e489106865241986f7f2ad28d4c8" /-! # Special shapes for limits in `Type`. The general shape (co)limits defined in `CategoryTheory.Limits.Types` are intended for use through the limits API, and the actual implementation should mostly be considered "sealed". In this file, we provide definitions of the "standard" special shapes of limits in `Type`, giving the expected definitional implementation: * the terminal object is `PUnit` * the binary product of `X` and `Y` is `X × Y` * the product of a family `f : J → Type` is `Π j, f j` * the coproduct of a family `f : J → Type` is `Σ j, f j` * the binary coproduct of `X` and `Y` is the sum type `X ⊕ Y` * the equalizer of a pair of maps `(g, h)` is the subtype `{x : Y // g x = h x}` * the coequalizer of a pair of maps `(f, g)` is the quotient of `Y` by `∀ x : Y, f x ~ g x` * the pullback of `f : X ⟶ Z` and `g : Y ⟶ Z` is the subtype `{ p : X × Y // f p.1 = g p.2 }` of the product We first construct terms of `IsLimit` and `LimitCone`, and then provide isomorphisms with the types generated by the `HasLimit` API. As an example, when setting up the monoidal category structure on `Type` we use the `Types.terminalLimitCone` and `Types.binaryProductLimitCone` definitions. -/ universe v u open CategoryTheory Limits namespace CategoryTheory.Limits.Types example : HasProducts.{v} (Type v) := inferInstance example [UnivLE.{v, u}] : HasProducts.{v} (Type u) := inferInstance -- This shortcut instance is required in `Mathlib.CategoryTheory.Closed.Types`, -- although I don't understand why, and wish it wasn't. instance : HasProducts.{v} (Type v) := inferInstance /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`. -/ @[simp 1001] theorem pi_lift_π_apply {β : Type v} [Small.{u} β] (f : β → Type u) {P : Type u} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := congr_fun (limit.lift_π (Fan.mk P s) ⟨b⟩) x #align category_theory.limits.types.pi_lift_π_apply CategoryTheory.Limits.Types.pi_lift_π_apply /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`, with specialized universes. -/ theorem pi_lift_π_apply' {β : Type v} (f : β → Type v) {P : Type v} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := by simp #align category_theory.limits.types.pi_lift_π_apply' CategoryTheory.Limits.Types.pi_lift_π_apply' /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`. -/ @[simp 1001] theorem pi_map_π_apply {β : Type v} [Small.{u} β] {f g : β → Type u} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := Limit.map_π_apply.{v, u} _ _ _ #align category_theory.limits.types.pi_map_π_apply CategoryTheory.Limits.Types.pi_map_π_apply /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`, with specialized universes. -/ theorem pi_map_π_apply' {β : Type v} {f g : β → Type v} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := by simp #align category_theory.limits.types.pi_map_π_apply' CategoryTheory.Limits.Types.pi_map_π_apply' /-- The category of types has `PUnit` as a terminal object. -/ def terminalLimitCone : Limits.LimitCone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cone := { pt := PUnit π := (Functor.uniqueFromEmpty _).hom } isLimit := { lift := fun _ _ => PUnit.unit fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext apply Subsingleton.elim } #align category_theory.limits.types.terminal_limit_cone CategoryTheory.Limits.Types.terminalLimitCone /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def terminalIso : ⊤_ Type u ≅ PUnit := limit.isoLimitCone terminalLimitCone.{u, 0} #align category_theory.limits.types.terminal_iso CategoryTheory.Limits.Types.terminalIso /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def isTerminalPunit : IsTerminal (PUnit : Type u) := terminalIsTerminal.ofIso terminalIso #align category_theory.limits.types.is_terminal_punit CategoryTheory.Limits.Types.isTerminalPunit -- porting note: the following three instances have been added to ease -- the automation in a definition in `AlgebraicTopology.SimplicialSet` noncomputable instance : Inhabited (⊤_ (Type u)) := ⟨@terminal.from (Type u) _ _ (ULift (Fin 1)) (ULift.up 0)⟩ instance : Subsingleton (⊤_ (Type u)) := ⟨fun a b => congr_fun (@Subsingleton.elim (_ ⟶ ⊤_ (Type u)) _ (fun _ => a) (fun _ => b)) (ULift.up (0 : Fin 1))⟩ noncomputable instance : Unique (⊤_ (Type u)) := Unique.mk' _ /-- A type is terminal if and only if it contains exactly one element. -/ noncomputable def isTerminalEquivUnique (X : Type u) : IsTerminal X ≃ Unique X := equivOfSubsingletonOfSubsingleton (fun h => ((Iso.toEquiv (terminalIsoIsTerminal h).symm).unique)) (fun _ => IsTerminal.ofIso terminalIsTerminal (Equiv.toIso (Equiv.equivOfUnique _ _))) /-- A type is terminal if and only if it is isomorphic to `PUnit`. -/ noncomputable def isTerminalEquivIsoPUnit (X : Type u) : IsTerminal X ≃ (X ≅ PUnit) := by calc IsTerminal X ≃ Unique X := isTerminalEquivUnique _ _ ≃ (X ≃ PUnit.{u + 1}) := uniqueEquivEquivUnique _ _ _ ≃ (X ≅ PUnit) := equivEquivIso /-- The category of types has `PEmpty` as an initial object. -/ def initialColimitCocone : Limits.ColimitCocone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cocone := { pt := PEmpty ι := (Functor.uniqueFromEmpty _).inv } isColimit := { desc := fun _ => by rintro ⟨⟩ fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext x;
cases x
/-- The category of types has `PEmpty` as an initial object. -/ def initialColimitCocone : Limits.ColimitCocone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cocone := { pt := PEmpty ι := (Functor.uniqueFromEmpty _).inv } isColimit := { desc := fun _ => by rintro ⟨⟩ fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext x;
Mathlib.CategoryTheory.Limits.Shapes.Types.134_0.ctQAUYXLRXnvMGw
/-- The category of types has `PEmpty` as an initial object. -/ def initialColimitCocone : Limits.ColimitCocone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cocone
Mathlib_CategoryTheory_Limits_Shapes_Types
⊢ binaryProductFunctor ≅ prod.functor
/- Copyright (c) 2020 Scott Morrison. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Scott Morrison -/ import Mathlib.CategoryTheory.Limits.Types import Mathlib.CategoryTheory.Limits.Shapes.Products import Mathlib.CategoryTheory.Limits.Shapes.BinaryProducts import Mathlib.CategoryTheory.Limits.Shapes.Terminal import Mathlib.CategoryTheory.ConcreteCategory.Basic import Mathlib.Tactic.CategoryTheory.Elementwise #align_import category_theory.limits.shapes.types from "leanprover-community/mathlib"@"5dc6092d09e5e489106865241986f7f2ad28d4c8" /-! # Special shapes for limits in `Type`. The general shape (co)limits defined in `CategoryTheory.Limits.Types` are intended for use through the limits API, and the actual implementation should mostly be considered "sealed". In this file, we provide definitions of the "standard" special shapes of limits in `Type`, giving the expected definitional implementation: * the terminal object is `PUnit` * the binary product of `X` and `Y` is `X × Y` * the product of a family `f : J → Type` is `Π j, f j` * the coproduct of a family `f : J → Type` is `Σ j, f j` * the binary coproduct of `X` and `Y` is the sum type `X ⊕ Y` * the equalizer of a pair of maps `(g, h)` is the subtype `{x : Y // g x = h x}` * the coequalizer of a pair of maps `(f, g)` is the quotient of `Y` by `∀ x : Y, f x ~ g x` * the pullback of `f : X ⟶ Z` and `g : Y ⟶ Z` is the subtype `{ p : X × Y // f p.1 = g p.2 }` of the product We first construct terms of `IsLimit` and `LimitCone`, and then provide isomorphisms with the types generated by the `HasLimit` API. As an example, when setting up the monoidal category structure on `Type` we use the `Types.terminalLimitCone` and `Types.binaryProductLimitCone` definitions. -/ universe v u open CategoryTheory Limits namespace CategoryTheory.Limits.Types example : HasProducts.{v} (Type v) := inferInstance example [UnivLE.{v, u}] : HasProducts.{v} (Type u) := inferInstance -- This shortcut instance is required in `Mathlib.CategoryTheory.Closed.Types`, -- although I don't understand why, and wish it wasn't. instance : HasProducts.{v} (Type v) := inferInstance /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`. -/ @[simp 1001] theorem pi_lift_π_apply {β : Type v} [Small.{u} β] (f : β → Type u) {P : Type u} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := congr_fun (limit.lift_π (Fan.mk P s) ⟨b⟩) x #align category_theory.limits.types.pi_lift_π_apply CategoryTheory.Limits.Types.pi_lift_π_apply /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`, with specialized universes. -/ theorem pi_lift_π_apply' {β : Type v} (f : β → Type v) {P : Type v} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := by simp #align category_theory.limits.types.pi_lift_π_apply' CategoryTheory.Limits.Types.pi_lift_π_apply' /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`. -/ @[simp 1001] theorem pi_map_π_apply {β : Type v} [Small.{u} β] {f g : β → Type u} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := Limit.map_π_apply.{v, u} _ _ _ #align category_theory.limits.types.pi_map_π_apply CategoryTheory.Limits.Types.pi_map_π_apply /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`, with specialized universes. -/ theorem pi_map_π_apply' {β : Type v} {f g : β → Type v} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := by simp #align category_theory.limits.types.pi_map_π_apply' CategoryTheory.Limits.Types.pi_map_π_apply' /-- The category of types has `PUnit` as a terminal object. -/ def terminalLimitCone : Limits.LimitCone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cone := { pt := PUnit π := (Functor.uniqueFromEmpty _).hom } isLimit := { lift := fun _ _ => PUnit.unit fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext apply Subsingleton.elim } #align category_theory.limits.types.terminal_limit_cone CategoryTheory.Limits.Types.terminalLimitCone /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def terminalIso : ⊤_ Type u ≅ PUnit := limit.isoLimitCone terminalLimitCone.{u, 0} #align category_theory.limits.types.terminal_iso CategoryTheory.Limits.Types.terminalIso /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def isTerminalPunit : IsTerminal (PUnit : Type u) := terminalIsTerminal.ofIso terminalIso #align category_theory.limits.types.is_terminal_punit CategoryTheory.Limits.Types.isTerminalPunit -- porting note: the following three instances have been added to ease -- the automation in a definition in `AlgebraicTopology.SimplicialSet` noncomputable instance : Inhabited (⊤_ (Type u)) := ⟨@terminal.from (Type u) _ _ (ULift (Fin 1)) (ULift.up 0)⟩ instance : Subsingleton (⊤_ (Type u)) := ⟨fun a b => congr_fun (@Subsingleton.elim (_ ⟶ ⊤_ (Type u)) _ (fun _ => a) (fun _ => b)) (ULift.up (0 : Fin 1))⟩ noncomputable instance : Unique (⊤_ (Type u)) := Unique.mk' _ /-- A type is terminal if and only if it contains exactly one element. -/ noncomputable def isTerminalEquivUnique (X : Type u) : IsTerminal X ≃ Unique X := equivOfSubsingletonOfSubsingleton (fun h => ((Iso.toEquiv (terminalIsoIsTerminal h).symm).unique)) (fun _ => IsTerminal.ofIso terminalIsTerminal (Equiv.toIso (Equiv.equivOfUnique _ _))) /-- A type is terminal if and only if it is isomorphic to `PUnit`. -/ noncomputable def isTerminalEquivIsoPUnit (X : Type u) : IsTerminal X ≃ (X ≅ PUnit) := by calc IsTerminal X ≃ Unique X := isTerminalEquivUnique _ _ ≃ (X ≃ PUnit.{u + 1}) := uniqueEquivEquivUnique _ _ _ ≃ (X ≅ PUnit) := equivEquivIso /-- The category of types has `PEmpty` as an initial object. -/ def initialColimitCocone : Limits.ColimitCocone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cocone := { pt := PEmpty ι := (Functor.uniqueFromEmpty _).inv } isColimit := { desc := fun _ => by rintro ⟨⟩ fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext x; cases x } #align category_theory.limits.types.initial_colimit_cocone CategoryTheory.Limits.Types.initialColimitCocone /-- The initial object in `Type u` is `PEmpty`. -/ noncomputable def initialIso : ⊥_ Type u ≅ PEmpty := colimit.isoColimitCocone initialColimitCocone.{u, 0} #align category_theory.limits.types.initial_iso CategoryTheory.Limits.Types.initialIso /-- The initial object in `Type u` is `PEmpty`. -/ noncomputable def isInitialPunit : IsInitial (PEmpty : Type u) := initialIsInitial.ofIso initialIso #align category_theory.limits.types.is_initial_punit CategoryTheory.Limits.Types.isInitialPunit open CategoryTheory.Limits.WalkingPair -- We manually generate the other projection lemmas since the simp-normal form for the legs is -- otherwise not created correctly. /-- The product type `X × Y` forms a cone for the binary product of `X` and `Y`. -/ @[simps! pt] def binaryProductCone (X Y : Type u) : BinaryFan X Y := BinaryFan.mk _root_.Prod.fst _root_.Prod.snd #align category_theory.limits.types.binary_product_cone CategoryTheory.Limits.Types.binaryProductCone @[simp] theorem binaryProductCone_fst (X Y : Type u) : (binaryProductCone X Y).fst = _root_.Prod.fst := rfl #align category_theory.limits.types.binary_product_cone_fst CategoryTheory.Limits.Types.binaryProductCone_fst @[simp] theorem binaryProductCone_snd (X Y : Type u) : (binaryProductCone X Y).snd = _root_.Prod.snd := rfl #align category_theory.limits.types.binary_product_cone_snd CategoryTheory.Limits.Types.binaryProductCone_snd /-- The product type `X × Y` is a binary product for `X` and `Y`. -/ @[simps] def binaryProductLimit (X Y : Type u) : IsLimit (binaryProductCone X Y) where lift (s : BinaryFan X Y) x := (s.fst x, s.snd x) fac _ j := Discrete.recOn j fun j => WalkingPair.casesOn j rfl rfl uniq _ _ w := funext fun x => Prod.ext (congr_fun (w ⟨left⟩) x) (congr_fun (w ⟨right⟩) x) #align category_theory.limits.types.binary_product_limit CategoryTheory.Limits.Types.binaryProductLimit /-- The category of types has `X × Y`, the usual cartesian product, as the binary product of `X` and `Y`. -/ @[simps] def binaryProductLimitCone (X Y : Type u) : Limits.LimitCone (pair X Y) := ⟨_, binaryProductLimit X Y⟩ #align category_theory.limits.types.binary_product_limit_cone CategoryTheory.Limits.Types.binaryProductLimitCone /-- The categorical binary product in `Type u` is cartesian product. -/ noncomputable def binaryProductIso (X Y : Type u) : Limits.prod X Y ≅ X × Y := limit.isoLimitCone (binaryProductLimitCone X Y) #align category_theory.limits.types.binary_product_iso CategoryTheory.Limits.Types.binaryProductIso @[elementwise (attr := simp)] theorem binaryProductIso_hom_comp_fst (X Y : Type u) : (binaryProductIso X Y).hom ≫ _root_.Prod.fst = Limits.prod.fst := limit.isoLimitCone_hom_π (binaryProductLimitCone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_product_iso_hom_comp_fst CategoryTheory.Limits.Types.binaryProductIso_hom_comp_fst @[elementwise (attr := simp)] theorem binaryProductIso_hom_comp_snd (X Y : Type u) : (binaryProductIso X Y).hom ≫ _root_.Prod.snd = Limits.prod.snd := limit.isoLimitCone_hom_π (binaryProductLimitCone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_product_iso_hom_comp_snd CategoryTheory.Limits.Types.binaryProductIso_hom_comp_snd @[elementwise (attr := simp)] theorem binaryProductIso_inv_comp_fst (X Y : Type u) : (binaryProductIso X Y).inv ≫ Limits.prod.fst = _root_.Prod.fst := limit.isoLimitCone_inv_π (binaryProductLimitCone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_product_iso_inv_comp_fst CategoryTheory.Limits.Types.binaryProductIso_inv_comp_fst @[elementwise (attr := simp)] theorem binaryProductIso_inv_comp_snd (X Y : Type u) : (binaryProductIso X Y).inv ≫ Limits.prod.snd = _root_.Prod.snd := limit.isoLimitCone_inv_π (binaryProductLimitCone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_product_iso_inv_comp_snd CategoryTheory.Limits.Types.binaryProductIso_inv_comp_snd -- porting note: it was originally @[simps (config := { typeMd := reducible })] -- We add the option `type_md` to tell `@[simps]` to not treat homomorphisms `X ⟶ Y` in `Type*` as -- a function type /-- The functor which sends `X, Y` to the product type `X × Y`. -/ @[simps] def binaryProductFunctor : Type u ⥤ Type u ⥤ Type u where obj X := { obj := fun Y => X × Y map := fun { Y₁ Y₂} f => (binaryProductLimit X Y₂).lift (BinaryFan.mk _root_.Prod.fst (_root_.Prod.snd ≫ f)) } map {X₁ X₂} f := { app := fun Y => (binaryProductLimit X₂ Y).lift (BinaryFan.mk (_root_.Prod.fst ≫ f) _root_.Prod.snd) } #align category_theory.limits.types.binary_product_functor CategoryTheory.Limits.Types.binaryProductFunctor /-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _) := by
refine' NatIso.ofComponents (fun X => _) (fun _ => _)
/-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _) := by
Mathlib.CategoryTheory.Limits.Shapes.Types.236_0.ctQAUYXLRXnvMGw
/-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _)
Mathlib_CategoryTheory_Limits_Shapes_Types
case refine'_1 X : Type u ⊢ binaryProductFunctor.obj X ≅ prod.functor.obj X
/- Copyright (c) 2020 Scott Morrison. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Scott Morrison -/ import Mathlib.CategoryTheory.Limits.Types import Mathlib.CategoryTheory.Limits.Shapes.Products import Mathlib.CategoryTheory.Limits.Shapes.BinaryProducts import Mathlib.CategoryTheory.Limits.Shapes.Terminal import Mathlib.CategoryTheory.ConcreteCategory.Basic import Mathlib.Tactic.CategoryTheory.Elementwise #align_import category_theory.limits.shapes.types from "leanprover-community/mathlib"@"5dc6092d09e5e489106865241986f7f2ad28d4c8" /-! # Special shapes for limits in `Type`. The general shape (co)limits defined in `CategoryTheory.Limits.Types` are intended for use through the limits API, and the actual implementation should mostly be considered "sealed". In this file, we provide definitions of the "standard" special shapes of limits in `Type`, giving the expected definitional implementation: * the terminal object is `PUnit` * the binary product of `X` and `Y` is `X × Y` * the product of a family `f : J → Type` is `Π j, f j` * the coproduct of a family `f : J → Type` is `Σ j, f j` * the binary coproduct of `X` and `Y` is the sum type `X ⊕ Y` * the equalizer of a pair of maps `(g, h)` is the subtype `{x : Y // g x = h x}` * the coequalizer of a pair of maps `(f, g)` is the quotient of `Y` by `∀ x : Y, f x ~ g x` * the pullback of `f : X ⟶ Z` and `g : Y ⟶ Z` is the subtype `{ p : X × Y // f p.1 = g p.2 }` of the product We first construct terms of `IsLimit` and `LimitCone`, and then provide isomorphisms with the types generated by the `HasLimit` API. As an example, when setting up the monoidal category structure on `Type` we use the `Types.terminalLimitCone` and `Types.binaryProductLimitCone` definitions. -/ universe v u open CategoryTheory Limits namespace CategoryTheory.Limits.Types example : HasProducts.{v} (Type v) := inferInstance example [UnivLE.{v, u}] : HasProducts.{v} (Type u) := inferInstance -- This shortcut instance is required in `Mathlib.CategoryTheory.Closed.Types`, -- although I don't understand why, and wish it wasn't. instance : HasProducts.{v} (Type v) := inferInstance /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`. -/ @[simp 1001] theorem pi_lift_π_apply {β : Type v} [Small.{u} β] (f : β → Type u) {P : Type u} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := congr_fun (limit.lift_π (Fan.mk P s) ⟨b⟩) x #align category_theory.limits.types.pi_lift_π_apply CategoryTheory.Limits.Types.pi_lift_π_apply /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`, with specialized universes. -/ theorem pi_lift_π_apply' {β : Type v} (f : β → Type v) {P : Type v} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := by simp #align category_theory.limits.types.pi_lift_π_apply' CategoryTheory.Limits.Types.pi_lift_π_apply' /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`. -/ @[simp 1001] theorem pi_map_π_apply {β : Type v} [Small.{u} β] {f g : β → Type u} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := Limit.map_π_apply.{v, u} _ _ _ #align category_theory.limits.types.pi_map_π_apply CategoryTheory.Limits.Types.pi_map_π_apply /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`, with specialized universes. -/ theorem pi_map_π_apply' {β : Type v} {f g : β → Type v} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := by simp #align category_theory.limits.types.pi_map_π_apply' CategoryTheory.Limits.Types.pi_map_π_apply' /-- The category of types has `PUnit` as a terminal object. -/ def terminalLimitCone : Limits.LimitCone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cone := { pt := PUnit π := (Functor.uniqueFromEmpty _).hom } isLimit := { lift := fun _ _ => PUnit.unit fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext apply Subsingleton.elim } #align category_theory.limits.types.terminal_limit_cone CategoryTheory.Limits.Types.terminalLimitCone /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def terminalIso : ⊤_ Type u ≅ PUnit := limit.isoLimitCone terminalLimitCone.{u, 0} #align category_theory.limits.types.terminal_iso CategoryTheory.Limits.Types.terminalIso /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def isTerminalPunit : IsTerminal (PUnit : Type u) := terminalIsTerminal.ofIso terminalIso #align category_theory.limits.types.is_terminal_punit CategoryTheory.Limits.Types.isTerminalPunit -- porting note: the following three instances have been added to ease -- the automation in a definition in `AlgebraicTopology.SimplicialSet` noncomputable instance : Inhabited (⊤_ (Type u)) := ⟨@terminal.from (Type u) _ _ (ULift (Fin 1)) (ULift.up 0)⟩ instance : Subsingleton (⊤_ (Type u)) := ⟨fun a b => congr_fun (@Subsingleton.elim (_ ⟶ ⊤_ (Type u)) _ (fun _ => a) (fun _ => b)) (ULift.up (0 : Fin 1))⟩ noncomputable instance : Unique (⊤_ (Type u)) := Unique.mk' _ /-- A type is terminal if and only if it contains exactly one element. -/ noncomputable def isTerminalEquivUnique (X : Type u) : IsTerminal X ≃ Unique X := equivOfSubsingletonOfSubsingleton (fun h => ((Iso.toEquiv (terminalIsoIsTerminal h).symm).unique)) (fun _ => IsTerminal.ofIso terminalIsTerminal (Equiv.toIso (Equiv.equivOfUnique _ _))) /-- A type is terminal if and only if it is isomorphic to `PUnit`. -/ noncomputable def isTerminalEquivIsoPUnit (X : Type u) : IsTerminal X ≃ (X ≅ PUnit) := by calc IsTerminal X ≃ Unique X := isTerminalEquivUnique _ _ ≃ (X ≃ PUnit.{u + 1}) := uniqueEquivEquivUnique _ _ _ ≃ (X ≅ PUnit) := equivEquivIso /-- The category of types has `PEmpty` as an initial object. -/ def initialColimitCocone : Limits.ColimitCocone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cocone := { pt := PEmpty ι := (Functor.uniqueFromEmpty _).inv } isColimit := { desc := fun _ => by rintro ⟨⟩ fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext x; cases x } #align category_theory.limits.types.initial_colimit_cocone CategoryTheory.Limits.Types.initialColimitCocone /-- The initial object in `Type u` is `PEmpty`. -/ noncomputable def initialIso : ⊥_ Type u ≅ PEmpty := colimit.isoColimitCocone initialColimitCocone.{u, 0} #align category_theory.limits.types.initial_iso CategoryTheory.Limits.Types.initialIso /-- The initial object in `Type u` is `PEmpty`. -/ noncomputable def isInitialPunit : IsInitial (PEmpty : Type u) := initialIsInitial.ofIso initialIso #align category_theory.limits.types.is_initial_punit CategoryTheory.Limits.Types.isInitialPunit open CategoryTheory.Limits.WalkingPair -- We manually generate the other projection lemmas since the simp-normal form for the legs is -- otherwise not created correctly. /-- The product type `X × Y` forms a cone for the binary product of `X` and `Y`. -/ @[simps! pt] def binaryProductCone (X Y : Type u) : BinaryFan X Y := BinaryFan.mk _root_.Prod.fst _root_.Prod.snd #align category_theory.limits.types.binary_product_cone CategoryTheory.Limits.Types.binaryProductCone @[simp] theorem binaryProductCone_fst (X Y : Type u) : (binaryProductCone X Y).fst = _root_.Prod.fst := rfl #align category_theory.limits.types.binary_product_cone_fst CategoryTheory.Limits.Types.binaryProductCone_fst @[simp] theorem binaryProductCone_snd (X Y : Type u) : (binaryProductCone X Y).snd = _root_.Prod.snd := rfl #align category_theory.limits.types.binary_product_cone_snd CategoryTheory.Limits.Types.binaryProductCone_snd /-- The product type `X × Y` is a binary product for `X` and `Y`. -/ @[simps] def binaryProductLimit (X Y : Type u) : IsLimit (binaryProductCone X Y) where lift (s : BinaryFan X Y) x := (s.fst x, s.snd x) fac _ j := Discrete.recOn j fun j => WalkingPair.casesOn j rfl rfl uniq _ _ w := funext fun x => Prod.ext (congr_fun (w ⟨left⟩) x) (congr_fun (w ⟨right⟩) x) #align category_theory.limits.types.binary_product_limit CategoryTheory.Limits.Types.binaryProductLimit /-- The category of types has `X × Y`, the usual cartesian product, as the binary product of `X` and `Y`. -/ @[simps] def binaryProductLimitCone (X Y : Type u) : Limits.LimitCone (pair X Y) := ⟨_, binaryProductLimit X Y⟩ #align category_theory.limits.types.binary_product_limit_cone CategoryTheory.Limits.Types.binaryProductLimitCone /-- The categorical binary product in `Type u` is cartesian product. -/ noncomputable def binaryProductIso (X Y : Type u) : Limits.prod X Y ≅ X × Y := limit.isoLimitCone (binaryProductLimitCone X Y) #align category_theory.limits.types.binary_product_iso CategoryTheory.Limits.Types.binaryProductIso @[elementwise (attr := simp)] theorem binaryProductIso_hom_comp_fst (X Y : Type u) : (binaryProductIso X Y).hom ≫ _root_.Prod.fst = Limits.prod.fst := limit.isoLimitCone_hom_π (binaryProductLimitCone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_product_iso_hom_comp_fst CategoryTheory.Limits.Types.binaryProductIso_hom_comp_fst @[elementwise (attr := simp)] theorem binaryProductIso_hom_comp_snd (X Y : Type u) : (binaryProductIso X Y).hom ≫ _root_.Prod.snd = Limits.prod.snd := limit.isoLimitCone_hom_π (binaryProductLimitCone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_product_iso_hom_comp_snd CategoryTheory.Limits.Types.binaryProductIso_hom_comp_snd @[elementwise (attr := simp)] theorem binaryProductIso_inv_comp_fst (X Y : Type u) : (binaryProductIso X Y).inv ≫ Limits.prod.fst = _root_.Prod.fst := limit.isoLimitCone_inv_π (binaryProductLimitCone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_product_iso_inv_comp_fst CategoryTheory.Limits.Types.binaryProductIso_inv_comp_fst @[elementwise (attr := simp)] theorem binaryProductIso_inv_comp_snd (X Y : Type u) : (binaryProductIso X Y).inv ≫ Limits.prod.snd = _root_.Prod.snd := limit.isoLimitCone_inv_π (binaryProductLimitCone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_product_iso_inv_comp_snd CategoryTheory.Limits.Types.binaryProductIso_inv_comp_snd -- porting note: it was originally @[simps (config := { typeMd := reducible })] -- We add the option `type_md` to tell `@[simps]` to not treat homomorphisms `X ⟶ Y` in `Type*` as -- a function type /-- The functor which sends `X, Y` to the product type `X × Y`. -/ @[simps] def binaryProductFunctor : Type u ⥤ Type u ⥤ Type u where obj X := { obj := fun Y => X × Y map := fun { Y₁ Y₂} f => (binaryProductLimit X Y₂).lift (BinaryFan.mk _root_.Prod.fst (_root_.Prod.snd ≫ f)) } map {X₁ X₂} f := { app := fun Y => (binaryProductLimit X₂ Y).lift (BinaryFan.mk (_root_.Prod.fst ≫ f) _root_.Prod.snd) } #align category_theory.limits.types.binary_product_functor CategoryTheory.Limits.Types.binaryProductFunctor /-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _) := by refine' NatIso.ofComponents (fun X => _) (fun _ => _) ·
refine' NatIso.ofComponents (fun Y => _) (fun _ => _)
/-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _) := by refine' NatIso.ofComponents (fun X => _) (fun _ => _) ·
Mathlib.CategoryTheory.Limits.Shapes.Types.236_0.ctQAUYXLRXnvMGw
/-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _)
Mathlib_CategoryTheory_Limits_Shapes_Types
case refine'_1.refine'_1 X Y : Type u ⊢ (binaryProductFunctor.obj X).obj Y ≅ (prod.functor.obj X).obj Y
/- Copyright (c) 2020 Scott Morrison. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Scott Morrison -/ import Mathlib.CategoryTheory.Limits.Types import Mathlib.CategoryTheory.Limits.Shapes.Products import Mathlib.CategoryTheory.Limits.Shapes.BinaryProducts import Mathlib.CategoryTheory.Limits.Shapes.Terminal import Mathlib.CategoryTheory.ConcreteCategory.Basic import Mathlib.Tactic.CategoryTheory.Elementwise #align_import category_theory.limits.shapes.types from "leanprover-community/mathlib"@"5dc6092d09e5e489106865241986f7f2ad28d4c8" /-! # Special shapes for limits in `Type`. The general shape (co)limits defined in `CategoryTheory.Limits.Types` are intended for use through the limits API, and the actual implementation should mostly be considered "sealed". In this file, we provide definitions of the "standard" special shapes of limits in `Type`, giving the expected definitional implementation: * the terminal object is `PUnit` * the binary product of `X` and `Y` is `X × Y` * the product of a family `f : J → Type` is `Π j, f j` * the coproduct of a family `f : J → Type` is `Σ j, f j` * the binary coproduct of `X` and `Y` is the sum type `X ⊕ Y` * the equalizer of a pair of maps `(g, h)` is the subtype `{x : Y // g x = h x}` * the coequalizer of a pair of maps `(f, g)` is the quotient of `Y` by `∀ x : Y, f x ~ g x` * the pullback of `f : X ⟶ Z` and `g : Y ⟶ Z` is the subtype `{ p : X × Y // f p.1 = g p.2 }` of the product We first construct terms of `IsLimit` and `LimitCone`, and then provide isomorphisms with the types generated by the `HasLimit` API. As an example, when setting up the monoidal category structure on `Type` we use the `Types.terminalLimitCone` and `Types.binaryProductLimitCone` definitions. -/ universe v u open CategoryTheory Limits namespace CategoryTheory.Limits.Types example : HasProducts.{v} (Type v) := inferInstance example [UnivLE.{v, u}] : HasProducts.{v} (Type u) := inferInstance -- This shortcut instance is required in `Mathlib.CategoryTheory.Closed.Types`, -- although I don't understand why, and wish it wasn't. instance : HasProducts.{v} (Type v) := inferInstance /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`. -/ @[simp 1001] theorem pi_lift_π_apply {β : Type v} [Small.{u} β] (f : β → Type u) {P : Type u} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := congr_fun (limit.lift_π (Fan.mk P s) ⟨b⟩) x #align category_theory.limits.types.pi_lift_π_apply CategoryTheory.Limits.Types.pi_lift_π_apply /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`, with specialized universes. -/ theorem pi_lift_π_apply' {β : Type v} (f : β → Type v) {P : Type v} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := by simp #align category_theory.limits.types.pi_lift_π_apply' CategoryTheory.Limits.Types.pi_lift_π_apply' /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`. -/ @[simp 1001] theorem pi_map_π_apply {β : Type v} [Small.{u} β] {f g : β → Type u} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := Limit.map_π_apply.{v, u} _ _ _ #align category_theory.limits.types.pi_map_π_apply CategoryTheory.Limits.Types.pi_map_π_apply /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`, with specialized universes. -/ theorem pi_map_π_apply' {β : Type v} {f g : β → Type v} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := by simp #align category_theory.limits.types.pi_map_π_apply' CategoryTheory.Limits.Types.pi_map_π_apply' /-- The category of types has `PUnit` as a terminal object. -/ def terminalLimitCone : Limits.LimitCone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cone := { pt := PUnit π := (Functor.uniqueFromEmpty _).hom } isLimit := { lift := fun _ _ => PUnit.unit fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext apply Subsingleton.elim } #align category_theory.limits.types.terminal_limit_cone CategoryTheory.Limits.Types.terminalLimitCone /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def terminalIso : ⊤_ Type u ≅ PUnit := limit.isoLimitCone terminalLimitCone.{u, 0} #align category_theory.limits.types.terminal_iso CategoryTheory.Limits.Types.terminalIso /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def isTerminalPunit : IsTerminal (PUnit : Type u) := terminalIsTerminal.ofIso terminalIso #align category_theory.limits.types.is_terminal_punit CategoryTheory.Limits.Types.isTerminalPunit -- porting note: the following three instances have been added to ease -- the automation in a definition in `AlgebraicTopology.SimplicialSet` noncomputable instance : Inhabited (⊤_ (Type u)) := ⟨@terminal.from (Type u) _ _ (ULift (Fin 1)) (ULift.up 0)⟩ instance : Subsingleton (⊤_ (Type u)) := ⟨fun a b => congr_fun (@Subsingleton.elim (_ ⟶ ⊤_ (Type u)) _ (fun _ => a) (fun _ => b)) (ULift.up (0 : Fin 1))⟩ noncomputable instance : Unique (⊤_ (Type u)) := Unique.mk' _ /-- A type is terminal if and only if it contains exactly one element. -/ noncomputable def isTerminalEquivUnique (X : Type u) : IsTerminal X ≃ Unique X := equivOfSubsingletonOfSubsingleton (fun h => ((Iso.toEquiv (terminalIsoIsTerminal h).symm).unique)) (fun _ => IsTerminal.ofIso terminalIsTerminal (Equiv.toIso (Equiv.equivOfUnique _ _))) /-- A type is terminal if and only if it is isomorphic to `PUnit`. -/ noncomputable def isTerminalEquivIsoPUnit (X : Type u) : IsTerminal X ≃ (X ≅ PUnit) := by calc IsTerminal X ≃ Unique X := isTerminalEquivUnique _ _ ≃ (X ≃ PUnit.{u + 1}) := uniqueEquivEquivUnique _ _ _ ≃ (X ≅ PUnit) := equivEquivIso /-- The category of types has `PEmpty` as an initial object. -/ def initialColimitCocone : Limits.ColimitCocone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cocone := { pt := PEmpty ι := (Functor.uniqueFromEmpty _).inv } isColimit := { desc := fun _ => by rintro ⟨⟩ fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext x; cases x } #align category_theory.limits.types.initial_colimit_cocone CategoryTheory.Limits.Types.initialColimitCocone /-- The initial object in `Type u` is `PEmpty`. -/ noncomputable def initialIso : ⊥_ Type u ≅ PEmpty := colimit.isoColimitCocone initialColimitCocone.{u, 0} #align category_theory.limits.types.initial_iso CategoryTheory.Limits.Types.initialIso /-- The initial object in `Type u` is `PEmpty`. -/ noncomputable def isInitialPunit : IsInitial (PEmpty : Type u) := initialIsInitial.ofIso initialIso #align category_theory.limits.types.is_initial_punit CategoryTheory.Limits.Types.isInitialPunit open CategoryTheory.Limits.WalkingPair -- We manually generate the other projection lemmas since the simp-normal form for the legs is -- otherwise not created correctly. /-- The product type `X × Y` forms a cone for the binary product of `X` and `Y`. -/ @[simps! pt] def binaryProductCone (X Y : Type u) : BinaryFan X Y := BinaryFan.mk _root_.Prod.fst _root_.Prod.snd #align category_theory.limits.types.binary_product_cone CategoryTheory.Limits.Types.binaryProductCone @[simp] theorem binaryProductCone_fst (X Y : Type u) : (binaryProductCone X Y).fst = _root_.Prod.fst := rfl #align category_theory.limits.types.binary_product_cone_fst CategoryTheory.Limits.Types.binaryProductCone_fst @[simp] theorem binaryProductCone_snd (X Y : Type u) : (binaryProductCone X Y).snd = _root_.Prod.snd := rfl #align category_theory.limits.types.binary_product_cone_snd CategoryTheory.Limits.Types.binaryProductCone_snd /-- The product type `X × Y` is a binary product for `X` and `Y`. -/ @[simps] def binaryProductLimit (X Y : Type u) : IsLimit (binaryProductCone X Y) where lift (s : BinaryFan X Y) x := (s.fst x, s.snd x) fac _ j := Discrete.recOn j fun j => WalkingPair.casesOn j rfl rfl uniq _ _ w := funext fun x => Prod.ext (congr_fun (w ⟨left⟩) x) (congr_fun (w ⟨right⟩) x) #align category_theory.limits.types.binary_product_limit CategoryTheory.Limits.Types.binaryProductLimit /-- The category of types has `X × Y`, the usual cartesian product, as the binary product of `X` and `Y`. -/ @[simps] def binaryProductLimitCone (X Y : Type u) : Limits.LimitCone (pair X Y) := ⟨_, binaryProductLimit X Y⟩ #align category_theory.limits.types.binary_product_limit_cone CategoryTheory.Limits.Types.binaryProductLimitCone /-- The categorical binary product in `Type u` is cartesian product. -/ noncomputable def binaryProductIso (X Y : Type u) : Limits.prod X Y ≅ X × Y := limit.isoLimitCone (binaryProductLimitCone X Y) #align category_theory.limits.types.binary_product_iso CategoryTheory.Limits.Types.binaryProductIso @[elementwise (attr := simp)] theorem binaryProductIso_hom_comp_fst (X Y : Type u) : (binaryProductIso X Y).hom ≫ _root_.Prod.fst = Limits.prod.fst := limit.isoLimitCone_hom_π (binaryProductLimitCone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_product_iso_hom_comp_fst CategoryTheory.Limits.Types.binaryProductIso_hom_comp_fst @[elementwise (attr := simp)] theorem binaryProductIso_hom_comp_snd (X Y : Type u) : (binaryProductIso X Y).hom ≫ _root_.Prod.snd = Limits.prod.snd := limit.isoLimitCone_hom_π (binaryProductLimitCone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_product_iso_hom_comp_snd CategoryTheory.Limits.Types.binaryProductIso_hom_comp_snd @[elementwise (attr := simp)] theorem binaryProductIso_inv_comp_fst (X Y : Type u) : (binaryProductIso X Y).inv ≫ Limits.prod.fst = _root_.Prod.fst := limit.isoLimitCone_inv_π (binaryProductLimitCone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_product_iso_inv_comp_fst CategoryTheory.Limits.Types.binaryProductIso_inv_comp_fst @[elementwise (attr := simp)] theorem binaryProductIso_inv_comp_snd (X Y : Type u) : (binaryProductIso X Y).inv ≫ Limits.prod.snd = _root_.Prod.snd := limit.isoLimitCone_inv_π (binaryProductLimitCone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_product_iso_inv_comp_snd CategoryTheory.Limits.Types.binaryProductIso_inv_comp_snd -- porting note: it was originally @[simps (config := { typeMd := reducible })] -- We add the option `type_md` to tell `@[simps]` to not treat homomorphisms `X ⟶ Y` in `Type*` as -- a function type /-- The functor which sends `X, Y` to the product type `X × Y`. -/ @[simps] def binaryProductFunctor : Type u ⥤ Type u ⥤ Type u where obj X := { obj := fun Y => X × Y map := fun { Y₁ Y₂} f => (binaryProductLimit X Y₂).lift (BinaryFan.mk _root_.Prod.fst (_root_.Prod.snd ≫ f)) } map {X₁ X₂} f := { app := fun Y => (binaryProductLimit X₂ Y).lift (BinaryFan.mk (_root_.Prod.fst ≫ f) _root_.Prod.snd) } #align category_theory.limits.types.binary_product_functor CategoryTheory.Limits.Types.binaryProductFunctor /-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _) := by refine' NatIso.ofComponents (fun X => _) (fun _ => _) · refine' NatIso.ofComponents (fun Y => _) (fun _ => _) ·
exact ((limit.isLimit _).conePointUniqueUpToIso (binaryProductLimit X Y)).symm
/-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _) := by refine' NatIso.ofComponents (fun X => _) (fun _ => _) · refine' NatIso.ofComponents (fun Y => _) (fun _ => _) ·
Mathlib.CategoryTheory.Limits.Shapes.Types.236_0.ctQAUYXLRXnvMGw
/-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _)
Mathlib_CategoryTheory_Limits_Shapes_Types
case refine'_1.refine'_2 X X✝ Y✝ : Type u x✝ : X✝ ⟶ Y✝ ⊢ (binaryProductFunctor.obj X).map x✝ ≫ ((fun Y => (IsLimit.conePointUniqueUpToIso (limit.isLimit (pair X Y)) (binaryProductLimit X Y)).symm) Y✝).hom = ((fun Y => (IsLimit.conePointUniqueUpToIso (limit.isLimit (pair X Y)) (binaryProductLimit X Y)).symm) X✝).hom ≫ (prod.functor.obj X).map x✝
/- Copyright (c) 2020 Scott Morrison. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Scott Morrison -/ import Mathlib.CategoryTheory.Limits.Types import Mathlib.CategoryTheory.Limits.Shapes.Products import Mathlib.CategoryTheory.Limits.Shapes.BinaryProducts import Mathlib.CategoryTheory.Limits.Shapes.Terminal import Mathlib.CategoryTheory.ConcreteCategory.Basic import Mathlib.Tactic.CategoryTheory.Elementwise #align_import category_theory.limits.shapes.types from "leanprover-community/mathlib"@"5dc6092d09e5e489106865241986f7f2ad28d4c8" /-! # Special shapes for limits in `Type`. The general shape (co)limits defined in `CategoryTheory.Limits.Types` are intended for use through the limits API, and the actual implementation should mostly be considered "sealed". In this file, we provide definitions of the "standard" special shapes of limits in `Type`, giving the expected definitional implementation: * the terminal object is `PUnit` * the binary product of `X` and `Y` is `X × Y` * the product of a family `f : J → Type` is `Π j, f j` * the coproduct of a family `f : J → Type` is `Σ j, f j` * the binary coproduct of `X` and `Y` is the sum type `X ⊕ Y` * the equalizer of a pair of maps `(g, h)` is the subtype `{x : Y // g x = h x}` * the coequalizer of a pair of maps `(f, g)` is the quotient of `Y` by `∀ x : Y, f x ~ g x` * the pullback of `f : X ⟶ Z` and `g : Y ⟶ Z` is the subtype `{ p : X × Y // f p.1 = g p.2 }` of the product We first construct terms of `IsLimit` and `LimitCone`, and then provide isomorphisms with the types generated by the `HasLimit` API. As an example, when setting up the monoidal category structure on `Type` we use the `Types.terminalLimitCone` and `Types.binaryProductLimitCone` definitions. -/ universe v u open CategoryTheory Limits namespace CategoryTheory.Limits.Types example : HasProducts.{v} (Type v) := inferInstance example [UnivLE.{v, u}] : HasProducts.{v} (Type u) := inferInstance -- This shortcut instance is required in `Mathlib.CategoryTheory.Closed.Types`, -- although I don't understand why, and wish it wasn't. instance : HasProducts.{v} (Type v) := inferInstance /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`. -/ @[simp 1001] theorem pi_lift_π_apply {β : Type v} [Small.{u} β] (f : β → Type u) {P : Type u} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := congr_fun (limit.lift_π (Fan.mk P s) ⟨b⟩) x #align category_theory.limits.types.pi_lift_π_apply CategoryTheory.Limits.Types.pi_lift_π_apply /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`, with specialized universes. -/ theorem pi_lift_π_apply' {β : Type v} (f : β → Type v) {P : Type v} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := by simp #align category_theory.limits.types.pi_lift_π_apply' CategoryTheory.Limits.Types.pi_lift_π_apply' /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`. -/ @[simp 1001] theorem pi_map_π_apply {β : Type v} [Small.{u} β] {f g : β → Type u} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := Limit.map_π_apply.{v, u} _ _ _ #align category_theory.limits.types.pi_map_π_apply CategoryTheory.Limits.Types.pi_map_π_apply /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`, with specialized universes. -/ theorem pi_map_π_apply' {β : Type v} {f g : β → Type v} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := by simp #align category_theory.limits.types.pi_map_π_apply' CategoryTheory.Limits.Types.pi_map_π_apply' /-- The category of types has `PUnit` as a terminal object. -/ def terminalLimitCone : Limits.LimitCone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cone := { pt := PUnit π := (Functor.uniqueFromEmpty _).hom } isLimit := { lift := fun _ _ => PUnit.unit fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext apply Subsingleton.elim } #align category_theory.limits.types.terminal_limit_cone CategoryTheory.Limits.Types.terminalLimitCone /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def terminalIso : ⊤_ Type u ≅ PUnit := limit.isoLimitCone terminalLimitCone.{u, 0} #align category_theory.limits.types.terminal_iso CategoryTheory.Limits.Types.terminalIso /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def isTerminalPunit : IsTerminal (PUnit : Type u) := terminalIsTerminal.ofIso terminalIso #align category_theory.limits.types.is_terminal_punit CategoryTheory.Limits.Types.isTerminalPunit -- porting note: the following three instances have been added to ease -- the automation in a definition in `AlgebraicTopology.SimplicialSet` noncomputable instance : Inhabited (⊤_ (Type u)) := ⟨@terminal.from (Type u) _ _ (ULift (Fin 1)) (ULift.up 0)⟩ instance : Subsingleton (⊤_ (Type u)) := ⟨fun a b => congr_fun (@Subsingleton.elim (_ ⟶ ⊤_ (Type u)) _ (fun _ => a) (fun _ => b)) (ULift.up (0 : Fin 1))⟩ noncomputable instance : Unique (⊤_ (Type u)) := Unique.mk' _ /-- A type is terminal if and only if it contains exactly one element. -/ noncomputable def isTerminalEquivUnique (X : Type u) : IsTerminal X ≃ Unique X := equivOfSubsingletonOfSubsingleton (fun h => ((Iso.toEquiv (terminalIsoIsTerminal h).symm).unique)) (fun _ => IsTerminal.ofIso terminalIsTerminal (Equiv.toIso (Equiv.equivOfUnique _ _))) /-- A type is terminal if and only if it is isomorphic to `PUnit`. -/ noncomputable def isTerminalEquivIsoPUnit (X : Type u) : IsTerminal X ≃ (X ≅ PUnit) := by calc IsTerminal X ≃ Unique X := isTerminalEquivUnique _ _ ≃ (X ≃ PUnit.{u + 1}) := uniqueEquivEquivUnique _ _ _ ≃ (X ≅ PUnit) := equivEquivIso /-- The category of types has `PEmpty` as an initial object. -/ def initialColimitCocone : Limits.ColimitCocone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cocone := { pt := PEmpty ι := (Functor.uniqueFromEmpty _).inv } isColimit := { desc := fun _ => by rintro ⟨⟩ fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext x; cases x } #align category_theory.limits.types.initial_colimit_cocone CategoryTheory.Limits.Types.initialColimitCocone /-- The initial object in `Type u` is `PEmpty`. -/ noncomputable def initialIso : ⊥_ Type u ≅ PEmpty := colimit.isoColimitCocone initialColimitCocone.{u, 0} #align category_theory.limits.types.initial_iso CategoryTheory.Limits.Types.initialIso /-- The initial object in `Type u` is `PEmpty`. -/ noncomputable def isInitialPunit : IsInitial (PEmpty : Type u) := initialIsInitial.ofIso initialIso #align category_theory.limits.types.is_initial_punit CategoryTheory.Limits.Types.isInitialPunit open CategoryTheory.Limits.WalkingPair -- We manually generate the other projection lemmas since the simp-normal form for the legs is -- otherwise not created correctly. /-- The product type `X × Y` forms a cone for the binary product of `X` and `Y`. -/ @[simps! pt] def binaryProductCone (X Y : Type u) : BinaryFan X Y := BinaryFan.mk _root_.Prod.fst _root_.Prod.snd #align category_theory.limits.types.binary_product_cone CategoryTheory.Limits.Types.binaryProductCone @[simp] theorem binaryProductCone_fst (X Y : Type u) : (binaryProductCone X Y).fst = _root_.Prod.fst := rfl #align category_theory.limits.types.binary_product_cone_fst CategoryTheory.Limits.Types.binaryProductCone_fst @[simp] theorem binaryProductCone_snd (X Y : Type u) : (binaryProductCone X Y).snd = _root_.Prod.snd := rfl #align category_theory.limits.types.binary_product_cone_snd CategoryTheory.Limits.Types.binaryProductCone_snd /-- The product type `X × Y` is a binary product for `X` and `Y`. -/ @[simps] def binaryProductLimit (X Y : Type u) : IsLimit (binaryProductCone X Y) where lift (s : BinaryFan X Y) x := (s.fst x, s.snd x) fac _ j := Discrete.recOn j fun j => WalkingPair.casesOn j rfl rfl uniq _ _ w := funext fun x => Prod.ext (congr_fun (w ⟨left⟩) x) (congr_fun (w ⟨right⟩) x) #align category_theory.limits.types.binary_product_limit CategoryTheory.Limits.Types.binaryProductLimit /-- The category of types has `X × Y`, the usual cartesian product, as the binary product of `X` and `Y`. -/ @[simps] def binaryProductLimitCone (X Y : Type u) : Limits.LimitCone (pair X Y) := ⟨_, binaryProductLimit X Y⟩ #align category_theory.limits.types.binary_product_limit_cone CategoryTheory.Limits.Types.binaryProductLimitCone /-- The categorical binary product in `Type u` is cartesian product. -/ noncomputable def binaryProductIso (X Y : Type u) : Limits.prod X Y ≅ X × Y := limit.isoLimitCone (binaryProductLimitCone X Y) #align category_theory.limits.types.binary_product_iso CategoryTheory.Limits.Types.binaryProductIso @[elementwise (attr := simp)] theorem binaryProductIso_hom_comp_fst (X Y : Type u) : (binaryProductIso X Y).hom ≫ _root_.Prod.fst = Limits.prod.fst := limit.isoLimitCone_hom_π (binaryProductLimitCone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_product_iso_hom_comp_fst CategoryTheory.Limits.Types.binaryProductIso_hom_comp_fst @[elementwise (attr := simp)] theorem binaryProductIso_hom_comp_snd (X Y : Type u) : (binaryProductIso X Y).hom ≫ _root_.Prod.snd = Limits.prod.snd := limit.isoLimitCone_hom_π (binaryProductLimitCone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_product_iso_hom_comp_snd CategoryTheory.Limits.Types.binaryProductIso_hom_comp_snd @[elementwise (attr := simp)] theorem binaryProductIso_inv_comp_fst (X Y : Type u) : (binaryProductIso X Y).inv ≫ Limits.prod.fst = _root_.Prod.fst := limit.isoLimitCone_inv_π (binaryProductLimitCone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_product_iso_inv_comp_fst CategoryTheory.Limits.Types.binaryProductIso_inv_comp_fst @[elementwise (attr := simp)] theorem binaryProductIso_inv_comp_snd (X Y : Type u) : (binaryProductIso X Y).inv ≫ Limits.prod.snd = _root_.Prod.snd := limit.isoLimitCone_inv_π (binaryProductLimitCone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_product_iso_inv_comp_snd CategoryTheory.Limits.Types.binaryProductIso_inv_comp_snd -- porting note: it was originally @[simps (config := { typeMd := reducible })] -- We add the option `type_md` to tell `@[simps]` to not treat homomorphisms `X ⟶ Y` in `Type*` as -- a function type /-- The functor which sends `X, Y` to the product type `X × Y`. -/ @[simps] def binaryProductFunctor : Type u ⥤ Type u ⥤ Type u where obj X := { obj := fun Y => X × Y map := fun { Y₁ Y₂} f => (binaryProductLimit X Y₂).lift (BinaryFan.mk _root_.Prod.fst (_root_.Prod.snd ≫ f)) } map {X₁ X₂} f := { app := fun Y => (binaryProductLimit X₂ Y).lift (BinaryFan.mk (_root_.Prod.fst ≫ f) _root_.Prod.snd) } #align category_theory.limits.types.binary_product_functor CategoryTheory.Limits.Types.binaryProductFunctor /-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _) := by refine' NatIso.ofComponents (fun X => _) (fun _ => _) · refine' NatIso.ofComponents (fun Y => _) (fun _ => _) · exact ((limit.isLimit _).conePointUniqueUpToIso (binaryProductLimit X Y)).symm ·
apply Limits.prod.hom_ext
/-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _) := by refine' NatIso.ofComponents (fun X => _) (fun _ => _) · refine' NatIso.ofComponents (fun Y => _) (fun _ => _) · exact ((limit.isLimit _).conePointUniqueUpToIso (binaryProductLimit X Y)).symm ·
Mathlib.CategoryTheory.Limits.Shapes.Types.236_0.ctQAUYXLRXnvMGw
/-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _)
Mathlib_CategoryTheory_Limits_Shapes_Types
case refine'_1.refine'_2.h₁ X X✝ Y✝ : Type u x✝ : X✝ ⟶ Y✝ ⊢ ((binaryProductFunctor.obj X).map x✝ ≫ ((fun Y => (IsLimit.conePointUniqueUpToIso (limit.isLimit (pair X Y)) (binaryProductLimit X Y)).symm) Y✝).hom) ≫ prod.fst = (((fun Y => (IsLimit.conePointUniqueUpToIso (limit.isLimit (pair X Y)) (binaryProductLimit X Y)).symm) X✝).hom ≫ (prod.functor.obj X).map x✝) ≫ prod.fst
/- Copyright (c) 2020 Scott Morrison. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Scott Morrison -/ import Mathlib.CategoryTheory.Limits.Types import Mathlib.CategoryTheory.Limits.Shapes.Products import Mathlib.CategoryTheory.Limits.Shapes.BinaryProducts import Mathlib.CategoryTheory.Limits.Shapes.Terminal import Mathlib.CategoryTheory.ConcreteCategory.Basic import Mathlib.Tactic.CategoryTheory.Elementwise #align_import category_theory.limits.shapes.types from "leanprover-community/mathlib"@"5dc6092d09e5e489106865241986f7f2ad28d4c8" /-! # Special shapes for limits in `Type`. The general shape (co)limits defined in `CategoryTheory.Limits.Types` are intended for use through the limits API, and the actual implementation should mostly be considered "sealed". In this file, we provide definitions of the "standard" special shapes of limits in `Type`, giving the expected definitional implementation: * the terminal object is `PUnit` * the binary product of `X` and `Y` is `X × Y` * the product of a family `f : J → Type` is `Π j, f j` * the coproduct of a family `f : J → Type` is `Σ j, f j` * the binary coproduct of `X` and `Y` is the sum type `X ⊕ Y` * the equalizer of a pair of maps `(g, h)` is the subtype `{x : Y // g x = h x}` * the coequalizer of a pair of maps `(f, g)` is the quotient of `Y` by `∀ x : Y, f x ~ g x` * the pullback of `f : X ⟶ Z` and `g : Y ⟶ Z` is the subtype `{ p : X × Y // f p.1 = g p.2 }` of the product We first construct terms of `IsLimit` and `LimitCone`, and then provide isomorphisms with the types generated by the `HasLimit` API. As an example, when setting up the monoidal category structure on `Type` we use the `Types.terminalLimitCone` and `Types.binaryProductLimitCone` definitions. -/ universe v u open CategoryTheory Limits namespace CategoryTheory.Limits.Types example : HasProducts.{v} (Type v) := inferInstance example [UnivLE.{v, u}] : HasProducts.{v} (Type u) := inferInstance -- This shortcut instance is required in `Mathlib.CategoryTheory.Closed.Types`, -- although I don't understand why, and wish it wasn't. instance : HasProducts.{v} (Type v) := inferInstance /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`. -/ @[simp 1001] theorem pi_lift_π_apply {β : Type v} [Small.{u} β] (f : β → Type u) {P : Type u} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := congr_fun (limit.lift_π (Fan.mk P s) ⟨b⟩) x #align category_theory.limits.types.pi_lift_π_apply CategoryTheory.Limits.Types.pi_lift_π_apply /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`, with specialized universes. -/ theorem pi_lift_π_apply' {β : Type v} (f : β → Type v) {P : Type v} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := by simp #align category_theory.limits.types.pi_lift_π_apply' CategoryTheory.Limits.Types.pi_lift_π_apply' /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`. -/ @[simp 1001] theorem pi_map_π_apply {β : Type v} [Small.{u} β] {f g : β → Type u} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := Limit.map_π_apply.{v, u} _ _ _ #align category_theory.limits.types.pi_map_π_apply CategoryTheory.Limits.Types.pi_map_π_apply /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`, with specialized universes. -/ theorem pi_map_π_apply' {β : Type v} {f g : β → Type v} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := by simp #align category_theory.limits.types.pi_map_π_apply' CategoryTheory.Limits.Types.pi_map_π_apply' /-- The category of types has `PUnit` as a terminal object. -/ def terminalLimitCone : Limits.LimitCone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cone := { pt := PUnit π := (Functor.uniqueFromEmpty _).hom } isLimit := { lift := fun _ _ => PUnit.unit fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext apply Subsingleton.elim } #align category_theory.limits.types.terminal_limit_cone CategoryTheory.Limits.Types.terminalLimitCone /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def terminalIso : ⊤_ Type u ≅ PUnit := limit.isoLimitCone terminalLimitCone.{u, 0} #align category_theory.limits.types.terminal_iso CategoryTheory.Limits.Types.terminalIso /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def isTerminalPunit : IsTerminal (PUnit : Type u) := terminalIsTerminal.ofIso terminalIso #align category_theory.limits.types.is_terminal_punit CategoryTheory.Limits.Types.isTerminalPunit -- porting note: the following three instances have been added to ease -- the automation in a definition in `AlgebraicTopology.SimplicialSet` noncomputable instance : Inhabited (⊤_ (Type u)) := ⟨@terminal.from (Type u) _ _ (ULift (Fin 1)) (ULift.up 0)⟩ instance : Subsingleton (⊤_ (Type u)) := ⟨fun a b => congr_fun (@Subsingleton.elim (_ ⟶ ⊤_ (Type u)) _ (fun _ => a) (fun _ => b)) (ULift.up (0 : Fin 1))⟩ noncomputable instance : Unique (⊤_ (Type u)) := Unique.mk' _ /-- A type is terminal if and only if it contains exactly one element. -/ noncomputable def isTerminalEquivUnique (X : Type u) : IsTerminal X ≃ Unique X := equivOfSubsingletonOfSubsingleton (fun h => ((Iso.toEquiv (terminalIsoIsTerminal h).symm).unique)) (fun _ => IsTerminal.ofIso terminalIsTerminal (Equiv.toIso (Equiv.equivOfUnique _ _))) /-- A type is terminal if and only if it is isomorphic to `PUnit`. -/ noncomputable def isTerminalEquivIsoPUnit (X : Type u) : IsTerminal X ≃ (X ≅ PUnit) := by calc IsTerminal X ≃ Unique X := isTerminalEquivUnique _ _ ≃ (X ≃ PUnit.{u + 1}) := uniqueEquivEquivUnique _ _ _ ≃ (X ≅ PUnit) := equivEquivIso /-- The category of types has `PEmpty` as an initial object. -/ def initialColimitCocone : Limits.ColimitCocone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cocone := { pt := PEmpty ι := (Functor.uniqueFromEmpty _).inv } isColimit := { desc := fun _ => by rintro ⟨⟩ fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext x; cases x } #align category_theory.limits.types.initial_colimit_cocone CategoryTheory.Limits.Types.initialColimitCocone /-- The initial object in `Type u` is `PEmpty`. -/ noncomputable def initialIso : ⊥_ Type u ≅ PEmpty := colimit.isoColimitCocone initialColimitCocone.{u, 0} #align category_theory.limits.types.initial_iso CategoryTheory.Limits.Types.initialIso /-- The initial object in `Type u` is `PEmpty`. -/ noncomputable def isInitialPunit : IsInitial (PEmpty : Type u) := initialIsInitial.ofIso initialIso #align category_theory.limits.types.is_initial_punit CategoryTheory.Limits.Types.isInitialPunit open CategoryTheory.Limits.WalkingPair -- We manually generate the other projection lemmas since the simp-normal form for the legs is -- otherwise not created correctly. /-- The product type `X × Y` forms a cone for the binary product of `X` and `Y`. -/ @[simps! pt] def binaryProductCone (X Y : Type u) : BinaryFan X Y := BinaryFan.mk _root_.Prod.fst _root_.Prod.snd #align category_theory.limits.types.binary_product_cone CategoryTheory.Limits.Types.binaryProductCone @[simp] theorem binaryProductCone_fst (X Y : Type u) : (binaryProductCone X Y).fst = _root_.Prod.fst := rfl #align category_theory.limits.types.binary_product_cone_fst CategoryTheory.Limits.Types.binaryProductCone_fst @[simp] theorem binaryProductCone_snd (X Y : Type u) : (binaryProductCone X Y).snd = _root_.Prod.snd := rfl #align category_theory.limits.types.binary_product_cone_snd CategoryTheory.Limits.Types.binaryProductCone_snd /-- The product type `X × Y` is a binary product for `X` and `Y`. -/ @[simps] def binaryProductLimit (X Y : Type u) : IsLimit (binaryProductCone X Y) where lift (s : BinaryFan X Y) x := (s.fst x, s.snd x) fac _ j := Discrete.recOn j fun j => WalkingPair.casesOn j rfl rfl uniq _ _ w := funext fun x => Prod.ext (congr_fun (w ⟨left⟩) x) (congr_fun (w ⟨right⟩) x) #align category_theory.limits.types.binary_product_limit CategoryTheory.Limits.Types.binaryProductLimit /-- The category of types has `X × Y`, the usual cartesian product, as the binary product of `X` and `Y`. -/ @[simps] def binaryProductLimitCone (X Y : Type u) : Limits.LimitCone (pair X Y) := ⟨_, binaryProductLimit X Y⟩ #align category_theory.limits.types.binary_product_limit_cone CategoryTheory.Limits.Types.binaryProductLimitCone /-- The categorical binary product in `Type u` is cartesian product. -/ noncomputable def binaryProductIso (X Y : Type u) : Limits.prod X Y ≅ X × Y := limit.isoLimitCone (binaryProductLimitCone X Y) #align category_theory.limits.types.binary_product_iso CategoryTheory.Limits.Types.binaryProductIso @[elementwise (attr := simp)] theorem binaryProductIso_hom_comp_fst (X Y : Type u) : (binaryProductIso X Y).hom ≫ _root_.Prod.fst = Limits.prod.fst := limit.isoLimitCone_hom_π (binaryProductLimitCone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_product_iso_hom_comp_fst CategoryTheory.Limits.Types.binaryProductIso_hom_comp_fst @[elementwise (attr := simp)] theorem binaryProductIso_hom_comp_snd (X Y : Type u) : (binaryProductIso X Y).hom ≫ _root_.Prod.snd = Limits.prod.snd := limit.isoLimitCone_hom_π (binaryProductLimitCone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_product_iso_hom_comp_snd CategoryTheory.Limits.Types.binaryProductIso_hom_comp_snd @[elementwise (attr := simp)] theorem binaryProductIso_inv_comp_fst (X Y : Type u) : (binaryProductIso X Y).inv ≫ Limits.prod.fst = _root_.Prod.fst := limit.isoLimitCone_inv_π (binaryProductLimitCone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_product_iso_inv_comp_fst CategoryTheory.Limits.Types.binaryProductIso_inv_comp_fst @[elementwise (attr := simp)] theorem binaryProductIso_inv_comp_snd (X Y : Type u) : (binaryProductIso X Y).inv ≫ Limits.prod.snd = _root_.Prod.snd := limit.isoLimitCone_inv_π (binaryProductLimitCone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_product_iso_inv_comp_snd CategoryTheory.Limits.Types.binaryProductIso_inv_comp_snd -- porting note: it was originally @[simps (config := { typeMd := reducible })] -- We add the option `type_md` to tell `@[simps]` to not treat homomorphisms `X ⟶ Y` in `Type*` as -- a function type /-- The functor which sends `X, Y` to the product type `X × Y`. -/ @[simps] def binaryProductFunctor : Type u ⥤ Type u ⥤ Type u where obj X := { obj := fun Y => X × Y map := fun { Y₁ Y₂} f => (binaryProductLimit X Y₂).lift (BinaryFan.mk _root_.Prod.fst (_root_.Prod.snd ≫ f)) } map {X₁ X₂} f := { app := fun Y => (binaryProductLimit X₂ Y).lift (BinaryFan.mk (_root_.Prod.fst ≫ f) _root_.Prod.snd) } #align category_theory.limits.types.binary_product_functor CategoryTheory.Limits.Types.binaryProductFunctor /-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _) := by refine' NatIso.ofComponents (fun X => _) (fun _ => _) · refine' NatIso.ofComponents (fun Y => _) (fun _ => _) · exact ((limit.isLimit _).conePointUniqueUpToIso (binaryProductLimit X Y)).symm · apply Limits.prod.hom_ext <;>
simp
/-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _) := by refine' NatIso.ofComponents (fun X => _) (fun _ => _) · refine' NatIso.ofComponents (fun Y => _) (fun _ => _) · exact ((limit.isLimit _).conePointUniqueUpToIso (binaryProductLimit X Y)).symm · apply Limits.prod.hom_ext <;>
Mathlib.CategoryTheory.Limits.Shapes.Types.236_0.ctQAUYXLRXnvMGw
/-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _)
Mathlib_CategoryTheory_Limits_Shapes_Types
case refine'_1.refine'_2.h₂ X X✝ Y✝ : Type u x✝ : X✝ ⟶ Y✝ ⊢ ((binaryProductFunctor.obj X).map x✝ ≫ ((fun Y => (IsLimit.conePointUniqueUpToIso (limit.isLimit (pair X Y)) (binaryProductLimit X Y)).symm) Y✝).hom) ≫ prod.snd = (((fun Y => (IsLimit.conePointUniqueUpToIso (limit.isLimit (pair X Y)) (binaryProductLimit X Y)).symm) X✝).hom ≫ (prod.functor.obj X).map x✝) ≫ prod.snd
/- Copyright (c) 2020 Scott Morrison. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Scott Morrison -/ import Mathlib.CategoryTheory.Limits.Types import Mathlib.CategoryTheory.Limits.Shapes.Products import Mathlib.CategoryTheory.Limits.Shapes.BinaryProducts import Mathlib.CategoryTheory.Limits.Shapes.Terminal import Mathlib.CategoryTheory.ConcreteCategory.Basic import Mathlib.Tactic.CategoryTheory.Elementwise #align_import category_theory.limits.shapes.types from "leanprover-community/mathlib"@"5dc6092d09e5e489106865241986f7f2ad28d4c8" /-! # Special shapes for limits in `Type`. The general shape (co)limits defined in `CategoryTheory.Limits.Types` are intended for use through the limits API, and the actual implementation should mostly be considered "sealed". In this file, we provide definitions of the "standard" special shapes of limits in `Type`, giving the expected definitional implementation: * the terminal object is `PUnit` * the binary product of `X` and `Y` is `X × Y` * the product of a family `f : J → Type` is `Π j, f j` * the coproduct of a family `f : J → Type` is `Σ j, f j` * the binary coproduct of `X` and `Y` is the sum type `X ⊕ Y` * the equalizer of a pair of maps `(g, h)` is the subtype `{x : Y // g x = h x}` * the coequalizer of a pair of maps `(f, g)` is the quotient of `Y` by `∀ x : Y, f x ~ g x` * the pullback of `f : X ⟶ Z` and `g : Y ⟶ Z` is the subtype `{ p : X × Y // f p.1 = g p.2 }` of the product We first construct terms of `IsLimit` and `LimitCone`, and then provide isomorphisms with the types generated by the `HasLimit` API. As an example, when setting up the monoidal category structure on `Type` we use the `Types.terminalLimitCone` and `Types.binaryProductLimitCone` definitions. -/ universe v u open CategoryTheory Limits namespace CategoryTheory.Limits.Types example : HasProducts.{v} (Type v) := inferInstance example [UnivLE.{v, u}] : HasProducts.{v} (Type u) := inferInstance -- This shortcut instance is required in `Mathlib.CategoryTheory.Closed.Types`, -- although I don't understand why, and wish it wasn't. instance : HasProducts.{v} (Type v) := inferInstance /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`. -/ @[simp 1001] theorem pi_lift_π_apply {β : Type v} [Small.{u} β] (f : β → Type u) {P : Type u} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := congr_fun (limit.lift_π (Fan.mk P s) ⟨b⟩) x #align category_theory.limits.types.pi_lift_π_apply CategoryTheory.Limits.Types.pi_lift_π_apply /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`, with specialized universes. -/ theorem pi_lift_π_apply' {β : Type v} (f : β → Type v) {P : Type v} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := by simp #align category_theory.limits.types.pi_lift_π_apply' CategoryTheory.Limits.Types.pi_lift_π_apply' /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`. -/ @[simp 1001] theorem pi_map_π_apply {β : Type v} [Small.{u} β] {f g : β → Type u} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := Limit.map_π_apply.{v, u} _ _ _ #align category_theory.limits.types.pi_map_π_apply CategoryTheory.Limits.Types.pi_map_π_apply /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`, with specialized universes. -/ theorem pi_map_π_apply' {β : Type v} {f g : β → Type v} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := by simp #align category_theory.limits.types.pi_map_π_apply' CategoryTheory.Limits.Types.pi_map_π_apply' /-- The category of types has `PUnit` as a terminal object. -/ def terminalLimitCone : Limits.LimitCone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cone := { pt := PUnit π := (Functor.uniqueFromEmpty _).hom } isLimit := { lift := fun _ _ => PUnit.unit fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext apply Subsingleton.elim } #align category_theory.limits.types.terminal_limit_cone CategoryTheory.Limits.Types.terminalLimitCone /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def terminalIso : ⊤_ Type u ≅ PUnit := limit.isoLimitCone terminalLimitCone.{u, 0} #align category_theory.limits.types.terminal_iso CategoryTheory.Limits.Types.terminalIso /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def isTerminalPunit : IsTerminal (PUnit : Type u) := terminalIsTerminal.ofIso terminalIso #align category_theory.limits.types.is_terminal_punit CategoryTheory.Limits.Types.isTerminalPunit -- porting note: the following three instances have been added to ease -- the automation in a definition in `AlgebraicTopology.SimplicialSet` noncomputable instance : Inhabited (⊤_ (Type u)) := ⟨@terminal.from (Type u) _ _ (ULift (Fin 1)) (ULift.up 0)⟩ instance : Subsingleton (⊤_ (Type u)) := ⟨fun a b => congr_fun (@Subsingleton.elim (_ ⟶ ⊤_ (Type u)) _ (fun _ => a) (fun _ => b)) (ULift.up (0 : Fin 1))⟩ noncomputable instance : Unique (⊤_ (Type u)) := Unique.mk' _ /-- A type is terminal if and only if it contains exactly one element. -/ noncomputable def isTerminalEquivUnique (X : Type u) : IsTerminal X ≃ Unique X := equivOfSubsingletonOfSubsingleton (fun h => ((Iso.toEquiv (terminalIsoIsTerminal h).symm).unique)) (fun _ => IsTerminal.ofIso terminalIsTerminal (Equiv.toIso (Equiv.equivOfUnique _ _))) /-- A type is terminal if and only if it is isomorphic to `PUnit`. -/ noncomputable def isTerminalEquivIsoPUnit (X : Type u) : IsTerminal X ≃ (X ≅ PUnit) := by calc IsTerminal X ≃ Unique X := isTerminalEquivUnique _ _ ≃ (X ≃ PUnit.{u + 1}) := uniqueEquivEquivUnique _ _ _ ≃ (X ≅ PUnit) := equivEquivIso /-- The category of types has `PEmpty` as an initial object. -/ def initialColimitCocone : Limits.ColimitCocone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cocone := { pt := PEmpty ι := (Functor.uniqueFromEmpty _).inv } isColimit := { desc := fun _ => by rintro ⟨⟩ fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext x; cases x } #align category_theory.limits.types.initial_colimit_cocone CategoryTheory.Limits.Types.initialColimitCocone /-- The initial object in `Type u` is `PEmpty`. -/ noncomputable def initialIso : ⊥_ Type u ≅ PEmpty := colimit.isoColimitCocone initialColimitCocone.{u, 0} #align category_theory.limits.types.initial_iso CategoryTheory.Limits.Types.initialIso /-- The initial object in `Type u` is `PEmpty`. -/ noncomputable def isInitialPunit : IsInitial (PEmpty : Type u) := initialIsInitial.ofIso initialIso #align category_theory.limits.types.is_initial_punit CategoryTheory.Limits.Types.isInitialPunit open CategoryTheory.Limits.WalkingPair -- We manually generate the other projection lemmas since the simp-normal form for the legs is -- otherwise not created correctly. /-- The product type `X × Y` forms a cone for the binary product of `X` and `Y`. -/ @[simps! pt] def binaryProductCone (X Y : Type u) : BinaryFan X Y := BinaryFan.mk _root_.Prod.fst _root_.Prod.snd #align category_theory.limits.types.binary_product_cone CategoryTheory.Limits.Types.binaryProductCone @[simp] theorem binaryProductCone_fst (X Y : Type u) : (binaryProductCone X Y).fst = _root_.Prod.fst := rfl #align category_theory.limits.types.binary_product_cone_fst CategoryTheory.Limits.Types.binaryProductCone_fst @[simp] theorem binaryProductCone_snd (X Y : Type u) : (binaryProductCone X Y).snd = _root_.Prod.snd := rfl #align category_theory.limits.types.binary_product_cone_snd CategoryTheory.Limits.Types.binaryProductCone_snd /-- The product type `X × Y` is a binary product for `X` and `Y`. -/ @[simps] def binaryProductLimit (X Y : Type u) : IsLimit (binaryProductCone X Y) where lift (s : BinaryFan X Y) x := (s.fst x, s.snd x) fac _ j := Discrete.recOn j fun j => WalkingPair.casesOn j rfl rfl uniq _ _ w := funext fun x => Prod.ext (congr_fun (w ⟨left⟩) x) (congr_fun (w ⟨right⟩) x) #align category_theory.limits.types.binary_product_limit CategoryTheory.Limits.Types.binaryProductLimit /-- The category of types has `X × Y`, the usual cartesian product, as the binary product of `X` and `Y`. -/ @[simps] def binaryProductLimitCone (X Y : Type u) : Limits.LimitCone (pair X Y) := ⟨_, binaryProductLimit X Y⟩ #align category_theory.limits.types.binary_product_limit_cone CategoryTheory.Limits.Types.binaryProductLimitCone /-- The categorical binary product in `Type u` is cartesian product. -/ noncomputable def binaryProductIso (X Y : Type u) : Limits.prod X Y ≅ X × Y := limit.isoLimitCone (binaryProductLimitCone X Y) #align category_theory.limits.types.binary_product_iso CategoryTheory.Limits.Types.binaryProductIso @[elementwise (attr := simp)] theorem binaryProductIso_hom_comp_fst (X Y : Type u) : (binaryProductIso X Y).hom ≫ _root_.Prod.fst = Limits.prod.fst := limit.isoLimitCone_hom_π (binaryProductLimitCone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_product_iso_hom_comp_fst CategoryTheory.Limits.Types.binaryProductIso_hom_comp_fst @[elementwise (attr := simp)] theorem binaryProductIso_hom_comp_snd (X Y : Type u) : (binaryProductIso X Y).hom ≫ _root_.Prod.snd = Limits.prod.snd := limit.isoLimitCone_hom_π (binaryProductLimitCone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_product_iso_hom_comp_snd CategoryTheory.Limits.Types.binaryProductIso_hom_comp_snd @[elementwise (attr := simp)] theorem binaryProductIso_inv_comp_fst (X Y : Type u) : (binaryProductIso X Y).inv ≫ Limits.prod.fst = _root_.Prod.fst := limit.isoLimitCone_inv_π (binaryProductLimitCone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_product_iso_inv_comp_fst CategoryTheory.Limits.Types.binaryProductIso_inv_comp_fst @[elementwise (attr := simp)] theorem binaryProductIso_inv_comp_snd (X Y : Type u) : (binaryProductIso X Y).inv ≫ Limits.prod.snd = _root_.Prod.snd := limit.isoLimitCone_inv_π (binaryProductLimitCone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_product_iso_inv_comp_snd CategoryTheory.Limits.Types.binaryProductIso_inv_comp_snd -- porting note: it was originally @[simps (config := { typeMd := reducible })] -- We add the option `type_md` to tell `@[simps]` to not treat homomorphisms `X ⟶ Y` in `Type*` as -- a function type /-- The functor which sends `X, Y` to the product type `X × Y`. -/ @[simps] def binaryProductFunctor : Type u ⥤ Type u ⥤ Type u where obj X := { obj := fun Y => X × Y map := fun { Y₁ Y₂} f => (binaryProductLimit X Y₂).lift (BinaryFan.mk _root_.Prod.fst (_root_.Prod.snd ≫ f)) } map {X₁ X₂} f := { app := fun Y => (binaryProductLimit X₂ Y).lift (BinaryFan.mk (_root_.Prod.fst ≫ f) _root_.Prod.snd) } #align category_theory.limits.types.binary_product_functor CategoryTheory.Limits.Types.binaryProductFunctor /-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _) := by refine' NatIso.ofComponents (fun X => _) (fun _ => _) · refine' NatIso.ofComponents (fun Y => _) (fun _ => _) · exact ((limit.isLimit _).conePointUniqueUpToIso (binaryProductLimit X Y)).symm · apply Limits.prod.hom_ext <;>
simp
/-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _) := by refine' NatIso.ofComponents (fun X => _) (fun _ => _) · refine' NatIso.ofComponents (fun Y => _) (fun _ => _) · exact ((limit.isLimit _).conePointUniqueUpToIso (binaryProductLimit X Y)).symm · apply Limits.prod.hom_ext <;>
Mathlib.CategoryTheory.Limits.Shapes.Types.236_0.ctQAUYXLRXnvMGw
/-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _)
Mathlib_CategoryTheory_Limits_Shapes_Types
case refine'_1.refine'_2.h₁ X X✝ Y✝ : Type u x✝ : X✝ ⟶ Y✝ ⊢ (binaryProductFunctor.obj X).map x✝ ≫ _root_.Prod.fst = _root_.Prod.fst
/- Copyright (c) 2020 Scott Morrison. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Scott Morrison -/ import Mathlib.CategoryTheory.Limits.Types import Mathlib.CategoryTheory.Limits.Shapes.Products import Mathlib.CategoryTheory.Limits.Shapes.BinaryProducts import Mathlib.CategoryTheory.Limits.Shapes.Terminal import Mathlib.CategoryTheory.ConcreteCategory.Basic import Mathlib.Tactic.CategoryTheory.Elementwise #align_import category_theory.limits.shapes.types from "leanprover-community/mathlib"@"5dc6092d09e5e489106865241986f7f2ad28d4c8" /-! # Special shapes for limits in `Type`. The general shape (co)limits defined in `CategoryTheory.Limits.Types` are intended for use through the limits API, and the actual implementation should mostly be considered "sealed". In this file, we provide definitions of the "standard" special shapes of limits in `Type`, giving the expected definitional implementation: * the terminal object is `PUnit` * the binary product of `X` and `Y` is `X × Y` * the product of a family `f : J → Type` is `Π j, f j` * the coproduct of a family `f : J → Type` is `Σ j, f j` * the binary coproduct of `X` and `Y` is the sum type `X ⊕ Y` * the equalizer of a pair of maps `(g, h)` is the subtype `{x : Y // g x = h x}` * the coequalizer of a pair of maps `(f, g)` is the quotient of `Y` by `∀ x : Y, f x ~ g x` * the pullback of `f : X ⟶ Z` and `g : Y ⟶ Z` is the subtype `{ p : X × Y // f p.1 = g p.2 }` of the product We first construct terms of `IsLimit` and `LimitCone`, and then provide isomorphisms with the types generated by the `HasLimit` API. As an example, when setting up the monoidal category structure on `Type` we use the `Types.terminalLimitCone` and `Types.binaryProductLimitCone` definitions. -/ universe v u open CategoryTheory Limits namespace CategoryTheory.Limits.Types example : HasProducts.{v} (Type v) := inferInstance example [UnivLE.{v, u}] : HasProducts.{v} (Type u) := inferInstance -- This shortcut instance is required in `Mathlib.CategoryTheory.Closed.Types`, -- although I don't understand why, and wish it wasn't. instance : HasProducts.{v} (Type v) := inferInstance /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`. -/ @[simp 1001] theorem pi_lift_π_apply {β : Type v} [Small.{u} β] (f : β → Type u) {P : Type u} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := congr_fun (limit.lift_π (Fan.mk P s) ⟨b⟩) x #align category_theory.limits.types.pi_lift_π_apply CategoryTheory.Limits.Types.pi_lift_π_apply /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`, with specialized universes. -/ theorem pi_lift_π_apply' {β : Type v} (f : β → Type v) {P : Type v} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := by simp #align category_theory.limits.types.pi_lift_π_apply' CategoryTheory.Limits.Types.pi_lift_π_apply' /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`. -/ @[simp 1001] theorem pi_map_π_apply {β : Type v} [Small.{u} β] {f g : β → Type u} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := Limit.map_π_apply.{v, u} _ _ _ #align category_theory.limits.types.pi_map_π_apply CategoryTheory.Limits.Types.pi_map_π_apply /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`, with specialized universes. -/ theorem pi_map_π_apply' {β : Type v} {f g : β → Type v} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := by simp #align category_theory.limits.types.pi_map_π_apply' CategoryTheory.Limits.Types.pi_map_π_apply' /-- The category of types has `PUnit` as a terminal object. -/ def terminalLimitCone : Limits.LimitCone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cone := { pt := PUnit π := (Functor.uniqueFromEmpty _).hom } isLimit := { lift := fun _ _ => PUnit.unit fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext apply Subsingleton.elim } #align category_theory.limits.types.terminal_limit_cone CategoryTheory.Limits.Types.terminalLimitCone /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def terminalIso : ⊤_ Type u ≅ PUnit := limit.isoLimitCone terminalLimitCone.{u, 0} #align category_theory.limits.types.terminal_iso CategoryTheory.Limits.Types.terminalIso /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def isTerminalPunit : IsTerminal (PUnit : Type u) := terminalIsTerminal.ofIso terminalIso #align category_theory.limits.types.is_terminal_punit CategoryTheory.Limits.Types.isTerminalPunit -- porting note: the following three instances have been added to ease -- the automation in a definition in `AlgebraicTopology.SimplicialSet` noncomputable instance : Inhabited (⊤_ (Type u)) := ⟨@terminal.from (Type u) _ _ (ULift (Fin 1)) (ULift.up 0)⟩ instance : Subsingleton (⊤_ (Type u)) := ⟨fun a b => congr_fun (@Subsingleton.elim (_ ⟶ ⊤_ (Type u)) _ (fun _ => a) (fun _ => b)) (ULift.up (0 : Fin 1))⟩ noncomputable instance : Unique (⊤_ (Type u)) := Unique.mk' _ /-- A type is terminal if and only if it contains exactly one element. -/ noncomputable def isTerminalEquivUnique (X : Type u) : IsTerminal X ≃ Unique X := equivOfSubsingletonOfSubsingleton (fun h => ((Iso.toEquiv (terminalIsoIsTerminal h).symm).unique)) (fun _ => IsTerminal.ofIso terminalIsTerminal (Equiv.toIso (Equiv.equivOfUnique _ _))) /-- A type is terminal if and only if it is isomorphic to `PUnit`. -/ noncomputable def isTerminalEquivIsoPUnit (X : Type u) : IsTerminal X ≃ (X ≅ PUnit) := by calc IsTerminal X ≃ Unique X := isTerminalEquivUnique _ _ ≃ (X ≃ PUnit.{u + 1}) := uniqueEquivEquivUnique _ _ _ ≃ (X ≅ PUnit) := equivEquivIso /-- The category of types has `PEmpty` as an initial object. -/ def initialColimitCocone : Limits.ColimitCocone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cocone := { pt := PEmpty ι := (Functor.uniqueFromEmpty _).inv } isColimit := { desc := fun _ => by rintro ⟨⟩ fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext x; cases x } #align category_theory.limits.types.initial_colimit_cocone CategoryTheory.Limits.Types.initialColimitCocone /-- The initial object in `Type u` is `PEmpty`. -/ noncomputable def initialIso : ⊥_ Type u ≅ PEmpty := colimit.isoColimitCocone initialColimitCocone.{u, 0} #align category_theory.limits.types.initial_iso CategoryTheory.Limits.Types.initialIso /-- The initial object in `Type u` is `PEmpty`. -/ noncomputable def isInitialPunit : IsInitial (PEmpty : Type u) := initialIsInitial.ofIso initialIso #align category_theory.limits.types.is_initial_punit CategoryTheory.Limits.Types.isInitialPunit open CategoryTheory.Limits.WalkingPair -- We manually generate the other projection lemmas since the simp-normal form for the legs is -- otherwise not created correctly. /-- The product type `X × Y` forms a cone for the binary product of `X` and `Y`. -/ @[simps! pt] def binaryProductCone (X Y : Type u) : BinaryFan X Y := BinaryFan.mk _root_.Prod.fst _root_.Prod.snd #align category_theory.limits.types.binary_product_cone CategoryTheory.Limits.Types.binaryProductCone @[simp] theorem binaryProductCone_fst (X Y : Type u) : (binaryProductCone X Y).fst = _root_.Prod.fst := rfl #align category_theory.limits.types.binary_product_cone_fst CategoryTheory.Limits.Types.binaryProductCone_fst @[simp] theorem binaryProductCone_snd (X Y : Type u) : (binaryProductCone X Y).snd = _root_.Prod.snd := rfl #align category_theory.limits.types.binary_product_cone_snd CategoryTheory.Limits.Types.binaryProductCone_snd /-- The product type `X × Y` is a binary product for `X` and `Y`. -/ @[simps] def binaryProductLimit (X Y : Type u) : IsLimit (binaryProductCone X Y) where lift (s : BinaryFan X Y) x := (s.fst x, s.snd x) fac _ j := Discrete.recOn j fun j => WalkingPair.casesOn j rfl rfl uniq _ _ w := funext fun x => Prod.ext (congr_fun (w ⟨left⟩) x) (congr_fun (w ⟨right⟩) x) #align category_theory.limits.types.binary_product_limit CategoryTheory.Limits.Types.binaryProductLimit /-- The category of types has `X × Y`, the usual cartesian product, as the binary product of `X` and `Y`. -/ @[simps] def binaryProductLimitCone (X Y : Type u) : Limits.LimitCone (pair X Y) := ⟨_, binaryProductLimit X Y⟩ #align category_theory.limits.types.binary_product_limit_cone CategoryTheory.Limits.Types.binaryProductLimitCone /-- The categorical binary product in `Type u` is cartesian product. -/ noncomputable def binaryProductIso (X Y : Type u) : Limits.prod X Y ≅ X × Y := limit.isoLimitCone (binaryProductLimitCone X Y) #align category_theory.limits.types.binary_product_iso CategoryTheory.Limits.Types.binaryProductIso @[elementwise (attr := simp)] theorem binaryProductIso_hom_comp_fst (X Y : Type u) : (binaryProductIso X Y).hom ≫ _root_.Prod.fst = Limits.prod.fst := limit.isoLimitCone_hom_π (binaryProductLimitCone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_product_iso_hom_comp_fst CategoryTheory.Limits.Types.binaryProductIso_hom_comp_fst @[elementwise (attr := simp)] theorem binaryProductIso_hom_comp_snd (X Y : Type u) : (binaryProductIso X Y).hom ≫ _root_.Prod.snd = Limits.prod.snd := limit.isoLimitCone_hom_π (binaryProductLimitCone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_product_iso_hom_comp_snd CategoryTheory.Limits.Types.binaryProductIso_hom_comp_snd @[elementwise (attr := simp)] theorem binaryProductIso_inv_comp_fst (X Y : Type u) : (binaryProductIso X Y).inv ≫ Limits.prod.fst = _root_.Prod.fst := limit.isoLimitCone_inv_π (binaryProductLimitCone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_product_iso_inv_comp_fst CategoryTheory.Limits.Types.binaryProductIso_inv_comp_fst @[elementwise (attr := simp)] theorem binaryProductIso_inv_comp_snd (X Y : Type u) : (binaryProductIso X Y).inv ≫ Limits.prod.snd = _root_.Prod.snd := limit.isoLimitCone_inv_π (binaryProductLimitCone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_product_iso_inv_comp_snd CategoryTheory.Limits.Types.binaryProductIso_inv_comp_snd -- porting note: it was originally @[simps (config := { typeMd := reducible })] -- We add the option `type_md` to tell `@[simps]` to not treat homomorphisms `X ⟶ Y` in `Type*` as -- a function type /-- The functor which sends `X, Y` to the product type `X × Y`. -/ @[simps] def binaryProductFunctor : Type u ⥤ Type u ⥤ Type u where obj X := { obj := fun Y => X × Y map := fun { Y₁ Y₂} f => (binaryProductLimit X Y₂).lift (BinaryFan.mk _root_.Prod.fst (_root_.Prod.snd ≫ f)) } map {X₁ X₂} f := { app := fun Y => (binaryProductLimit X₂ Y).lift (BinaryFan.mk (_root_.Prod.fst ≫ f) _root_.Prod.snd) } #align category_theory.limits.types.binary_product_functor CategoryTheory.Limits.Types.binaryProductFunctor /-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _) := by refine' NatIso.ofComponents (fun X => _) (fun _ => _) · refine' NatIso.ofComponents (fun Y => _) (fun _ => _) · exact ((limit.isLimit _).conePointUniqueUpToIso (binaryProductLimit X Y)).symm · apply Limits.prod.hom_ext <;> simp <;>
rfl
/-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _) := by refine' NatIso.ofComponents (fun X => _) (fun _ => _) · refine' NatIso.ofComponents (fun Y => _) (fun _ => _) · exact ((limit.isLimit _).conePointUniqueUpToIso (binaryProductLimit X Y)).symm · apply Limits.prod.hom_ext <;> simp <;>
Mathlib.CategoryTheory.Limits.Shapes.Types.236_0.ctQAUYXLRXnvMGw
/-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _)
Mathlib_CategoryTheory_Limits_Shapes_Types
case refine'_1.refine'_2.h₂ X X✝ Y✝ : Type u x✝ : X✝ ⟶ Y✝ ⊢ (binaryProductFunctor.obj X).map x✝ ≫ _root_.Prod.snd = _root_.Prod.snd ≫ x✝
/- Copyright (c) 2020 Scott Morrison. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Scott Morrison -/ import Mathlib.CategoryTheory.Limits.Types import Mathlib.CategoryTheory.Limits.Shapes.Products import Mathlib.CategoryTheory.Limits.Shapes.BinaryProducts import Mathlib.CategoryTheory.Limits.Shapes.Terminal import Mathlib.CategoryTheory.ConcreteCategory.Basic import Mathlib.Tactic.CategoryTheory.Elementwise #align_import category_theory.limits.shapes.types from "leanprover-community/mathlib"@"5dc6092d09e5e489106865241986f7f2ad28d4c8" /-! # Special shapes for limits in `Type`. The general shape (co)limits defined in `CategoryTheory.Limits.Types` are intended for use through the limits API, and the actual implementation should mostly be considered "sealed". In this file, we provide definitions of the "standard" special shapes of limits in `Type`, giving the expected definitional implementation: * the terminal object is `PUnit` * the binary product of `X` and `Y` is `X × Y` * the product of a family `f : J → Type` is `Π j, f j` * the coproduct of a family `f : J → Type` is `Σ j, f j` * the binary coproduct of `X` and `Y` is the sum type `X ⊕ Y` * the equalizer of a pair of maps `(g, h)` is the subtype `{x : Y // g x = h x}` * the coequalizer of a pair of maps `(f, g)` is the quotient of `Y` by `∀ x : Y, f x ~ g x` * the pullback of `f : X ⟶ Z` and `g : Y ⟶ Z` is the subtype `{ p : X × Y // f p.1 = g p.2 }` of the product We first construct terms of `IsLimit` and `LimitCone`, and then provide isomorphisms with the types generated by the `HasLimit` API. As an example, when setting up the monoidal category structure on `Type` we use the `Types.terminalLimitCone` and `Types.binaryProductLimitCone` definitions. -/ universe v u open CategoryTheory Limits namespace CategoryTheory.Limits.Types example : HasProducts.{v} (Type v) := inferInstance example [UnivLE.{v, u}] : HasProducts.{v} (Type u) := inferInstance -- This shortcut instance is required in `Mathlib.CategoryTheory.Closed.Types`, -- although I don't understand why, and wish it wasn't. instance : HasProducts.{v} (Type v) := inferInstance /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`. -/ @[simp 1001] theorem pi_lift_π_apply {β : Type v} [Small.{u} β] (f : β → Type u) {P : Type u} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := congr_fun (limit.lift_π (Fan.mk P s) ⟨b⟩) x #align category_theory.limits.types.pi_lift_π_apply CategoryTheory.Limits.Types.pi_lift_π_apply /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`, with specialized universes. -/ theorem pi_lift_π_apply' {β : Type v} (f : β → Type v) {P : Type v} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := by simp #align category_theory.limits.types.pi_lift_π_apply' CategoryTheory.Limits.Types.pi_lift_π_apply' /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`. -/ @[simp 1001] theorem pi_map_π_apply {β : Type v} [Small.{u} β] {f g : β → Type u} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := Limit.map_π_apply.{v, u} _ _ _ #align category_theory.limits.types.pi_map_π_apply CategoryTheory.Limits.Types.pi_map_π_apply /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`, with specialized universes. -/ theorem pi_map_π_apply' {β : Type v} {f g : β → Type v} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := by simp #align category_theory.limits.types.pi_map_π_apply' CategoryTheory.Limits.Types.pi_map_π_apply' /-- The category of types has `PUnit` as a terminal object. -/ def terminalLimitCone : Limits.LimitCone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cone := { pt := PUnit π := (Functor.uniqueFromEmpty _).hom } isLimit := { lift := fun _ _ => PUnit.unit fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext apply Subsingleton.elim } #align category_theory.limits.types.terminal_limit_cone CategoryTheory.Limits.Types.terminalLimitCone /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def terminalIso : ⊤_ Type u ≅ PUnit := limit.isoLimitCone terminalLimitCone.{u, 0} #align category_theory.limits.types.terminal_iso CategoryTheory.Limits.Types.terminalIso /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def isTerminalPunit : IsTerminal (PUnit : Type u) := terminalIsTerminal.ofIso terminalIso #align category_theory.limits.types.is_terminal_punit CategoryTheory.Limits.Types.isTerminalPunit -- porting note: the following three instances have been added to ease -- the automation in a definition in `AlgebraicTopology.SimplicialSet` noncomputable instance : Inhabited (⊤_ (Type u)) := ⟨@terminal.from (Type u) _ _ (ULift (Fin 1)) (ULift.up 0)⟩ instance : Subsingleton (⊤_ (Type u)) := ⟨fun a b => congr_fun (@Subsingleton.elim (_ ⟶ ⊤_ (Type u)) _ (fun _ => a) (fun _ => b)) (ULift.up (0 : Fin 1))⟩ noncomputable instance : Unique (⊤_ (Type u)) := Unique.mk' _ /-- A type is terminal if and only if it contains exactly one element. -/ noncomputable def isTerminalEquivUnique (X : Type u) : IsTerminal X ≃ Unique X := equivOfSubsingletonOfSubsingleton (fun h => ((Iso.toEquiv (terminalIsoIsTerminal h).symm).unique)) (fun _ => IsTerminal.ofIso terminalIsTerminal (Equiv.toIso (Equiv.equivOfUnique _ _))) /-- A type is terminal if and only if it is isomorphic to `PUnit`. -/ noncomputable def isTerminalEquivIsoPUnit (X : Type u) : IsTerminal X ≃ (X ≅ PUnit) := by calc IsTerminal X ≃ Unique X := isTerminalEquivUnique _ _ ≃ (X ≃ PUnit.{u + 1}) := uniqueEquivEquivUnique _ _ _ ≃ (X ≅ PUnit) := equivEquivIso /-- The category of types has `PEmpty` as an initial object. -/ def initialColimitCocone : Limits.ColimitCocone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cocone := { pt := PEmpty ι := (Functor.uniqueFromEmpty _).inv } isColimit := { desc := fun _ => by rintro ⟨⟩ fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext x; cases x } #align category_theory.limits.types.initial_colimit_cocone CategoryTheory.Limits.Types.initialColimitCocone /-- The initial object in `Type u` is `PEmpty`. -/ noncomputable def initialIso : ⊥_ Type u ≅ PEmpty := colimit.isoColimitCocone initialColimitCocone.{u, 0} #align category_theory.limits.types.initial_iso CategoryTheory.Limits.Types.initialIso /-- The initial object in `Type u` is `PEmpty`. -/ noncomputable def isInitialPunit : IsInitial (PEmpty : Type u) := initialIsInitial.ofIso initialIso #align category_theory.limits.types.is_initial_punit CategoryTheory.Limits.Types.isInitialPunit open CategoryTheory.Limits.WalkingPair -- We manually generate the other projection lemmas since the simp-normal form for the legs is -- otherwise not created correctly. /-- The product type `X × Y` forms a cone for the binary product of `X` and `Y`. -/ @[simps! pt] def binaryProductCone (X Y : Type u) : BinaryFan X Y := BinaryFan.mk _root_.Prod.fst _root_.Prod.snd #align category_theory.limits.types.binary_product_cone CategoryTheory.Limits.Types.binaryProductCone @[simp] theorem binaryProductCone_fst (X Y : Type u) : (binaryProductCone X Y).fst = _root_.Prod.fst := rfl #align category_theory.limits.types.binary_product_cone_fst CategoryTheory.Limits.Types.binaryProductCone_fst @[simp] theorem binaryProductCone_snd (X Y : Type u) : (binaryProductCone X Y).snd = _root_.Prod.snd := rfl #align category_theory.limits.types.binary_product_cone_snd CategoryTheory.Limits.Types.binaryProductCone_snd /-- The product type `X × Y` is a binary product for `X` and `Y`. -/ @[simps] def binaryProductLimit (X Y : Type u) : IsLimit (binaryProductCone X Y) where lift (s : BinaryFan X Y) x := (s.fst x, s.snd x) fac _ j := Discrete.recOn j fun j => WalkingPair.casesOn j rfl rfl uniq _ _ w := funext fun x => Prod.ext (congr_fun (w ⟨left⟩) x) (congr_fun (w ⟨right⟩) x) #align category_theory.limits.types.binary_product_limit CategoryTheory.Limits.Types.binaryProductLimit /-- The category of types has `X × Y`, the usual cartesian product, as the binary product of `X` and `Y`. -/ @[simps] def binaryProductLimitCone (X Y : Type u) : Limits.LimitCone (pair X Y) := ⟨_, binaryProductLimit X Y⟩ #align category_theory.limits.types.binary_product_limit_cone CategoryTheory.Limits.Types.binaryProductLimitCone /-- The categorical binary product in `Type u` is cartesian product. -/ noncomputable def binaryProductIso (X Y : Type u) : Limits.prod X Y ≅ X × Y := limit.isoLimitCone (binaryProductLimitCone X Y) #align category_theory.limits.types.binary_product_iso CategoryTheory.Limits.Types.binaryProductIso @[elementwise (attr := simp)] theorem binaryProductIso_hom_comp_fst (X Y : Type u) : (binaryProductIso X Y).hom ≫ _root_.Prod.fst = Limits.prod.fst := limit.isoLimitCone_hom_π (binaryProductLimitCone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_product_iso_hom_comp_fst CategoryTheory.Limits.Types.binaryProductIso_hom_comp_fst @[elementwise (attr := simp)] theorem binaryProductIso_hom_comp_snd (X Y : Type u) : (binaryProductIso X Y).hom ≫ _root_.Prod.snd = Limits.prod.snd := limit.isoLimitCone_hom_π (binaryProductLimitCone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_product_iso_hom_comp_snd CategoryTheory.Limits.Types.binaryProductIso_hom_comp_snd @[elementwise (attr := simp)] theorem binaryProductIso_inv_comp_fst (X Y : Type u) : (binaryProductIso X Y).inv ≫ Limits.prod.fst = _root_.Prod.fst := limit.isoLimitCone_inv_π (binaryProductLimitCone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_product_iso_inv_comp_fst CategoryTheory.Limits.Types.binaryProductIso_inv_comp_fst @[elementwise (attr := simp)] theorem binaryProductIso_inv_comp_snd (X Y : Type u) : (binaryProductIso X Y).inv ≫ Limits.prod.snd = _root_.Prod.snd := limit.isoLimitCone_inv_π (binaryProductLimitCone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_product_iso_inv_comp_snd CategoryTheory.Limits.Types.binaryProductIso_inv_comp_snd -- porting note: it was originally @[simps (config := { typeMd := reducible })] -- We add the option `type_md` to tell `@[simps]` to not treat homomorphisms `X ⟶ Y` in `Type*` as -- a function type /-- The functor which sends `X, Y` to the product type `X × Y`. -/ @[simps] def binaryProductFunctor : Type u ⥤ Type u ⥤ Type u where obj X := { obj := fun Y => X × Y map := fun { Y₁ Y₂} f => (binaryProductLimit X Y₂).lift (BinaryFan.mk _root_.Prod.fst (_root_.Prod.snd ≫ f)) } map {X₁ X₂} f := { app := fun Y => (binaryProductLimit X₂ Y).lift (BinaryFan.mk (_root_.Prod.fst ≫ f) _root_.Prod.snd) } #align category_theory.limits.types.binary_product_functor CategoryTheory.Limits.Types.binaryProductFunctor /-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _) := by refine' NatIso.ofComponents (fun X => _) (fun _ => _) · refine' NatIso.ofComponents (fun Y => _) (fun _ => _) · exact ((limit.isLimit _).conePointUniqueUpToIso (binaryProductLimit X Y)).symm · apply Limits.prod.hom_ext <;> simp <;>
rfl
/-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _) := by refine' NatIso.ofComponents (fun X => _) (fun _ => _) · refine' NatIso.ofComponents (fun Y => _) (fun _ => _) · exact ((limit.isLimit _).conePointUniqueUpToIso (binaryProductLimit X Y)).symm · apply Limits.prod.hom_ext <;> simp <;>
Mathlib.CategoryTheory.Limits.Shapes.Types.236_0.ctQAUYXLRXnvMGw
/-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _)
Mathlib_CategoryTheory_Limits_Shapes_Types
case refine'_2 X✝ Y✝ : Type u x✝ : X✝ ⟶ Y✝ ⊢ binaryProductFunctor.map x✝ ≫ ((fun X => NatIso.ofComponents fun Y => (IsLimit.conePointUniqueUpToIso (limit.isLimit (pair X Y)) (binaryProductLimit X Y)).symm) Y✝).hom = ((fun X => NatIso.ofComponents fun Y => (IsLimit.conePointUniqueUpToIso (limit.isLimit (pair X Y)) (binaryProductLimit X Y)).symm) X✝).hom ≫ prod.functor.map x✝
/- Copyright (c) 2020 Scott Morrison. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Scott Morrison -/ import Mathlib.CategoryTheory.Limits.Types import Mathlib.CategoryTheory.Limits.Shapes.Products import Mathlib.CategoryTheory.Limits.Shapes.BinaryProducts import Mathlib.CategoryTheory.Limits.Shapes.Terminal import Mathlib.CategoryTheory.ConcreteCategory.Basic import Mathlib.Tactic.CategoryTheory.Elementwise #align_import category_theory.limits.shapes.types from "leanprover-community/mathlib"@"5dc6092d09e5e489106865241986f7f2ad28d4c8" /-! # Special shapes for limits in `Type`. The general shape (co)limits defined in `CategoryTheory.Limits.Types` are intended for use through the limits API, and the actual implementation should mostly be considered "sealed". In this file, we provide definitions of the "standard" special shapes of limits in `Type`, giving the expected definitional implementation: * the terminal object is `PUnit` * the binary product of `X` and `Y` is `X × Y` * the product of a family `f : J → Type` is `Π j, f j` * the coproduct of a family `f : J → Type` is `Σ j, f j` * the binary coproduct of `X` and `Y` is the sum type `X ⊕ Y` * the equalizer of a pair of maps `(g, h)` is the subtype `{x : Y // g x = h x}` * the coequalizer of a pair of maps `(f, g)` is the quotient of `Y` by `∀ x : Y, f x ~ g x` * the pullback of `f : X ⟶ Z` and `g : Y ⟶ Z` is the subtype `{ p : X × Y // f p.1 = g p.2 }` of the product We first construct terms of `IsLimit` and `LimitCone`, and then provide isomorphisms with the types generated by the `HasLimit` API. As an example, when setting up the monoidal category structure on `Type` we use the `Types.terminalLimitCone` and `Types.binaryProductLimitCone` definitions. -/ universe v u open CategoryTheory Limits namespace CategoryTheory.Limits.Types example : HasProducts.{v} (Type v) := inferInstance example [UnivLE.{v, u}] : HasProducts.{v} (Type u) := inferInstance -- This shortcut instance is required in `Mathlib.CategoryTheory.Closed.Types`, -- although I don't understand why, and wish it wasn't. instance : HasProducts.{v} (Type v) := inferInstance /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`. -/ @[simp 1001] theorem pi_lift_π_apply {β : Type v} [Small.{u} β] (f : β → Type u) {P : Type u} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := congr_fun (limit.lift_π (Fan.mk P s) ⟨b⟩) x #align category_theory.limits.types.pi_lift_π_apply CategoryTheory.Limits.Types.pi_lift_π_apply /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`, with specialized universes. -/ theorem pi_lift_π_apply' {β : Type v} (f : β → Type v) {P : Type v} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := by simp #align category_theory.limits.types.pi_lift_π_apply' CategoryTheory.Limits.Types.pi_lift_π_apply' /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`. -/ @[simp 1001] theorem pi_map_π_apply {β : Type v} [Small.{u} β] {f g : β → Type u} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := Limit.map_π_apply.{v, u} _ _ _ #align category_theory.limits.types.pi_map_π_apply CategoryTheory.Limits.Types.pi_map_π_apply /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`, with specialized universes. -/ theorem pi_map_π_apply' {β : Type v} {f g : β → Type v} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := by simp #align category_theory.limits.types.pi_map_π_apply' CategoryTheory.Limits.Types.pi_map_π_apply' /-- The category of types has `PUnit` as a terminal object. -/ def terminalLimitCone : Limits.LimitCone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cone := { pt := PUnit π := (Functor.uniqueFromEmpty _).hom } isLimit := { lift := fun _ _ => PUnit.unit fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext apply Subsingleton.elim } #align category_theory.limits.types.terminal_limit_cone CategoryTheory.Limits.Types.terminalLimitCone /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def terminalIso : ⊤_ Type u ≅ PUnit := limit.isoLimitCone terminalLimitCone.{u, 0} #align category_theory.limits.types.terminal_iso CategoryTheory.Limits.Types.terminalIso /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def isTerminalPunit : IsTerminal (PUnit : Type u) := terminalIsTerminal.ofIso terminalIso #align category_theory.limits.types.is_terminal_punit CategoryTheory.Limits.Types.isTerminalPunit -- porting note: the following three instances have been added to ease -- the automation in a definition in `AlgebraicTopology.SimplicialSet` noncomputable instance : Inhabited (⊤_ (Type u)) := ⟨@terminal.from (Type u) _ _ (ULift (Fin 1)) (ULift.up 0)⟩ instance : Subsingleton (⊤_ (Type u)) := ⟨fun a b => congr_fun (@Subsingleton.elim (_ ⟶ ⊤_ (Type u)) _ (fun _ => a) (fun _ => b)) (ULift.up (0 : Fin 1))⟩ noncomputable instance : Unique (⊤_ (Type u)) := Unique.mk' _ /-- A type is terminal if and only if it contains exactly one element. -/ noncomputable def isTerminalEquivUnique (X : Type u) : IsTerminal X ≃ Unique X := equivOfSubsingletonOfSubsingleton (fun h => ((Iso.toEquiv (terminalIsoIsTerminal h).symm).unique)) (fun _ => IsTerminal.ofIso terminalIsTerminal (Equiv.toIso (Equiv.equivOfUnique _ _))) /-- A type is terminal if and only if it is isomorphic to `PUnit`. -/ noncomputable def isTerminalEquivIsoPUnit (X : Type u) : IsTerminal X ≃ (X ≅ PUnit) := by calc IsTerminal X ≃ Unique X := isTerminalEquivUnique _ _ ≃ (X ≃ PUnit.{u + 1}) := uniqueEquivEquivUnique _ _ _ ≃ (X ≅ PUnit) := equivEquivIso /-- The category of types has `PEmpty` as an initial object. -/ def initialColimitCocone : Limits.ColimitCocone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cocone := { pt := PEmpty ι := (Functor.uniqueFromEmpty _).inv } isColimit := { desc := fun _ => by rintro ⟨⟩ fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext x; cases x } #align category_theory.limits.types.initial_colimit_cocone CategoryTheory.Limits.Types.initialColimitCocone /-- The initial object in `Type u` is `PEmpty`. -/ noncomputable def initialIso : ⊥_ Type u ≅ PEmpty := colimit.isoColimitCocone initialColimitCocone.{u, 0} #align category_theory.limits.types.initial_iso CategoryTheory.Limits.Types.initialIso /-- The initial object in `Type u` is `PEmpty`. -/ noncomputable def isInitialPunit : IsInitial (PEmpty : Type u) := initialIsInitial.ofIso initialIso #align category_theory.limits.types.is_initial_punit CategoryTheory.Limits.Types.isInitialPunit open CategoryTheory.Limits.WalkingPair -- We manually generate the other projection lemmas since the simp-normal form for the legs is -- otherwise not created correctly. /-- The product type `X × Y` forms a cone for the binary product of `X` and `Y`. -/ @[simps! pt] def binaryProductCone (X Y : Type u) : BinaryFan X Y := BinaryFan.mk _root_.Prod.fst _root_.Prod.snd #align category_theory.limits.types.binary_product_cone CategoryTheory.Limits.Types.binaryProductCone @[simp] theorem binaryProductCone_fst (X Y : Type u) : (binaryProductCone X Y).fst = _root_.Prod.fst := rfl #align category_theory.limits.types.binary_product_cone_fst CategoryTheory.Limits.Types.binaryProductCone_fst @[simp] theorem binaryProductCone_snd (X Y : Type u) : (binaryProductCone X Y).snd = _root_.Prod.snd := rfl #align category_theory.limits.types.binary_product_cone_snd CategoryTheory.Limits.Types.binaryProductCone_snd /-- The product type `X × Y` is a binary product for `X` and `Y`. -/ @[simps] def binaryProductLimit (X Y : Type u) : IsLimit (binaryProductCone X Y) where lift (s : BinaryFan X Y) x := (s.fst x, s.snd x) fac _ j := Discrete.recOn j fun j => WalkingPair.casesOn j rfl rfl uniq _ _ w := funext fun x => Prod.ext (congr_fun (w ⟨left⟩) x) (congr_fun (w ⟨right⟩) x) #align category_theory.limits.types.binary_product_limit CategoryTheory.Limits.Types.binaryProductLimit /-- The category of types has `X × Y`, the usual cartesian product, as the binary product of `X` and `Y`. -/ @[simps] def binaryProductLimitCone (X Y : Type u) : Limits.LimitCone (pair X Y) := ⟨_, binaryProductLimit X Y⟩ #align category_theory.limits.types.binary_product_limit_cone CategoryTheory.Limits.Types.binaryProductLimitCone /-- The categorical binary product in `Type u` is cartesian product. -/ noncomputable def binaryProductIso (X Y : Type u) : Limits.prod X Y ≅ X × Y := limit.isoLimitCone (binaryProductLimitCone X Y) #align category_theory.limits.types.binary_product_iso CategoryTheory.Limits.Types.binaryProductIso @[elementwise (attr := simp)] theorem binaryProductIso_hom_comp_fst (X Y : Type u) : (binaryProductIso X Y).hom ≫ _root_.Prod.fst = Limits.prod.fst := limit.isoLimitCone_hom_π (binaryProductLimitCone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_product_iso_hom_comp_fst CategoryTheory.Limits.Types.binaryProductIso_hom_comp_fst @[elementwise (attr := simp)] theorem binaryProductIso_hom_comp_snd (X Y : Type u) : (binaryProductIso X Y).hom ≫ _root_.Prod.snd = Limits.prod.snd := limit.isoLimitCone_hom_π (binaryProductLimitCone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_product_iso_hom_comp_snd CategoryTheory.Limits.Types.binaryProductIso_hom_comp_snd @[elementwise (attr := simp)] theorem binaryProductIso_inv_comp_fst (X Y : Type u) : (binaryProductIso X Y).inv ≫ Limits.prod.fst = _root_.Prod.fst := limit.isoLimitCone_inv_π (binaryProductLimitCone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_product_iso_inv_comp_fst CategoryTheory.Limits.Types.binaryProductIso_inv_comp_fst @[elementwise (attr := simp)] theorem binaryProductIso_inv_comp_snd (X Y : Type u) : (binaryProductIso X Y).inv ≫ Limits.prod.snd = _root_.Prod.snd := limit.isoLimitCone_inv_π (binaryProductLimitCone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_product_iso_inv_comp_snd CategoryTheory.Limits.Types.binaryProductIso_inv_comp_snd -- porting note: it was originally @[simps (config := { typeMd := reducible })] -- We add the option `type_md` to tell `@[simps]` to not treat homomorphisms `X ⟶ Y` in `Type*` as -- a function type /-- The functor which sends `X, Y` to the product type `X × Y`. -/ @[simps] def binaryProductFunctor : Type u ⥤ Type u ⥤ Type u where obj X := { obj := fun Y => X × Y map := fun { Y₁ Y₂} f => (binaryProductLimit X Y₂).lift (BinaryFan.mk _root_.Prod.fst (_root_.Prod.snd ≫ f)) } map {X₁ X₂} f := { app := fun Y => (binaryProductLimit X₂ Y).lift (BinaryFan.mk (_root_.Prod.fst ≫ f) _root_.Prod.snd) } #align category_theory.limits.types.binary_product_functor CategoryTheory.Limits.Types.binaryProductFunctor /-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _) := by refine' NatIso.ofComponents (fun X => _) (fun _ => _) · refine' NatIso.ofComponents (fun Y => _) (fun _ => _) · exact ((limit.isLimit _).conePointUniqueUpToIso (binaryProductLimit X Y)).symm · apply Limits.prod.hom_ext <;> simp <;> rfl ·
ext : 2
/-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _) := by refine' NatIso.ofComponents (fun X => _) (fun _ => _) · refine' NatIso.ofComponents (fun Y => _) (fun _ => _) · exact ((limit.isLimit _).conePointUniqueUpToIso (binaryProductLimit X Y)).symm · apply Limits.prod.hom_ext <;> simp <;> rfl ·
Mathlib.CategoryTheory.Limits.Shapes.Types.236_0.ctQAUYXLRXnvMGw
/-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _)
Mathlib_CategoryTheory_Limits_Shapes_Types
case refine'_2.w.h X✝ Y✝ : Type u x✝¹ : X✝ ⟶ Y✝ x✝ : Type u ⊢ (binaryProductFunctor.map x✝¹ ≫ ((fun X => NatIso.ofComponents fun Y => (IsLimit.conePointUniqueUpToIso (limit.isLimit (pair X Y)) (binaryProductLimit X Y)).symm) Y✝).hom).app x✝ = (((fun X => NatIso.ofComponents fun Y => (IsLimit.conePointUniqueUpToIso (limit.isLimit (pair X Y)) (binaryProductLimit X Y)).symm) X✝).hom ≫ prod.functor.map x✝¹).app x✝
/- Copyright (c) 2020 Scott Morrison. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Scott Morrison -/ import Mathlib.CategoryTheory.Limits.Types import Mathlib.CategoryTheory.Limits.Shapes.Products import Mathlib.CategoryTheory.Limits.Shapes.BinaryProducts import Mathlib.CategoryTheory.Limits.Shapes.Terminal import Mathlib.CategoryTheory.ConcreteCategory.Basic import Mathlib.Tactic.CategoryTheory.Elementwise #align_import category_theory.limits.shapes.types from "leanprover-community/mathlib"@"5dc6092d09e5e489106865241986f7f2ad28d4c8" /-! # Special shapes for limits in `Type`. The general shape (co)limits defined in `CategoryTheory.Limits.Types` are intended for use through the limits API, and the actual implementation should mostly be considered "sealed". In this file, we provide definitions of the "standard" special shapes of limits in `Type`, giving the expected definitional implementation: * the terminal object is `PUnit` * the binary product of `X` and `Y` is `X × Y` * the product of a family `f : J → Type` is `Π j, f j` * the coproduct of a family `f : J → Type` is `Σ j, f j` * the binary coproduct of `X` and `Y` is the sum type `X ⊕ Y` * the equalizer of a pair of maps `(g, h)` is the subtype `{x : Y // g x = h x}` * the coequalizer of a pair of maps `(f, g)` is the quotient of `Y` by `∀ x : Y, f x ~ g x` * the pullback of `f : X ⟶ Z` and `g : Y ⟶ Z` is the subtype `{ p : X × Y // f p.1 = g p.2 }` of the product We first construct terms of `IsLimit` and `LimitCone`, and then provide isomorphisms with the types generated by the `HasLimit` API. As an example, when setting up the monoidal category structure on `Type` we use the `Types.terminalLimitCone` and `Types.binaryProductLimitCone` definitions. -/ universe v u open CategoryTheory Limits namespace CategoryTheory.Limits.Types example : HasProducts.{v} (Type v) := inferInstance example [UnivLE.{v, u}] : HasProducts.{v} (Type u) := inferInstance -- This shortcut instance is required in `Mathlib.CategoryTheory.Closed.Types`, -- although I don't understand why, and wish it wasn't. instance : HasProducts.{v} (Type v) := inferInstance /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`. -/ @[simp 1001] theorem pi_lift_π_apply {β : Type v} [Small.{u} β] (f : β → Type u) {P : Type u} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := congr_fun (limit.lift_π (Fan.mk P s) ⟨b⟩) x #align category_theory.limits.types.pi_lift_π_apply CategoryTheory.Limits.Types.pi_lift_π_apply /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`, with specialized universes. -/ theorem pi_lift_π_apply' {β : Type v} (f : β → Type v) {P : Type v} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := by simp #align category_theory.limits.types.pi_lift_π_apply' CategoryTheory.Limits.Types.pi_lift_π_apply' /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`. -/ @[simp 1001] theorem pi_map_π_apply {β : Type v} [Small.{u} β] {f g : β → Type u} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := Limit.map_π_apply.{v, u} _ _ _ #align category_theory.limits.types.pi_map_π_apply CategoryTheory.Limits.Types.pi_map_π_apply /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`, with specialized universes. -/ theorem pi_map_π_apply' {β : Type v} {f g : β → Type v} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := by simp #align category_theory.limits.types.pi_map_π_apply' CategoryTheory.Limits.Types.pi_map_π_apply' /-- The category of types has `PUnit` as a terminal object. -/ def terminalLimitCone : Limits.LimitCone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cone := { pt := PUnit π := (Functor.uniqueFromEmpty _).hom } isLimit := { lift := fun _ _ => PUnit.unit fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext apply Subsingleton.elim } #align category_theory.limits.types.terminal_limit_cone CategoryTheory.Limits.Types.terminalLimitCone /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def terminalIso : ⊤_ Type u ≅ PUnit := limit.isoLimitCone terminalLimitCone.{u, 0} #align category_theory.limits.types.terminal_iso CategoryTheory.Limits.Types.terminalIso /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def isTerminalPunit : IsTerminal (PUnit : Type u) := terminalIsTerminal.ofIso terminalIso #align category_theory.limits.types.is_terminal_punit CategoryTheory.Limits.Types.isTerminalPunit -- porting note: the following three instances have been added to ease -- the automation in a definition in `AlgebraicTopology.SimplicialSet` noncomputable instance : Inhabited (⊤_ (Type u)) := ⟨@terminal.from (Type u) _ _ (ULift (Fin 1)) (ULift.up 0)⟩ instance : Subsingleton (⊤_ (Type u)) := ⟨fun a b => congr_fun (@Subsingleton.elim (_ ⟶ ⊤_ (Type u)) _ (fun _ => a) (fun _ => b)) (ULift.up (0 : Fin 1))⟩ noncomputable instance : Unique (⊤_ (Type u)) := Unique.mk' _ /-- A type is terminal if and only if it contains exactly one element. -/ noncomputable def isTerminalEquivUnique (X : Type u) : IsTerminal X ≃ Unique X := equivOfSubsingletonOfSubsingleton (fun h => ((Iso.toEquiv (terminalIsoIsTerminal h).symm).unique)) (fun _ => IsTerminal.ofIso terminalIsTerminal (Equiv.toIso (Equiv.equivOfUnique _ _))) /-- A type is terminal if and only if it is isomorphic to `PUnit`. -/ noncomputable def isTerminalEquivIsoPUnit (X : Type u) : IsTerminal X ≃ (X ≅ PUnit) := by calc IsTerminal X ≃ Unique X := isTerminalEquivUnique _ _ ≃ (X ≃ PUnit.{u + 1}) := uniqueEquivEquivUnique _ _ _ ≃ (X ≅ PUnit) := equivEquivIso /-- The category of types has `PEmpty` as an initial object. -/ def initialColimitCocone : Limits.ColimitCocone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cocone := { pt := PEmpty ι := (Functor.uniqueFromEmpty _).inv } isColimit := { desc := fun _ => by rintro ⟨⟩ fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext x; cases x } #align category_theory.limits.types.initial_colimit_cocone CategoryTheory.Limits.Types.initialColimitCocone /-- The initial object in `Type u` is `PEmpty`. -/ noncomputable def initialIso : ⊥_ Type u ≅ PEmpty := colimit.isoColimitCocone initialColimitCocone.{u, 0} #align category_theory.limits.types.initial_iso CategoryTheory.Limits.Types.initialIso /-- The initial object in `Type u` is `PEmpty`. -/ noncomputable def isInitialPunit : IsInitial (PEmpty : Type u) := initialIsInitial.ofIso initialIso #align category_theory.limits.types.is_initial_punit CategoryTheory.Limits.Types.isInitialPunit open CategoryTheory.Limits.WalkingPair -- We manually generate the other projection lemmas since the simp-normal form for the legs is -- otherwise not created correctly. /-- The product type `X × Y` forms a cone for the binary product of `X` and `Y`. -/ @[simps! pt] def binaryProductCone (X Y : Type u) : BinaryFan X Y := BinaryFan.mk _root_.Prod.fst _root_.Prod.snd #align category_theory.limits.types.binary_product_cone CategoryTheory.Limits.Types.binaryProductCone @[simp] theorem binaryProductCone_fst (X Y : Type u) : (binaryProductCone X Y).fst = _root_.Prod.fst := rfl #align category_theory.limits.types.binary_product_cone_fst CategoryTheory.Limits.Types.binaryProductCone_fst @[simp] theorem binaryProductCone_snd (X Y : Type u) : (binaryProductCone X Y).snd = _root_.Prod.snd := rfl #align category_theory.limits.types.binary_product_cone_snd CategoryTheory.Limits.Types.binaryProductCone_snd /-- The product type `X × Y` is a binary product for `X` and `Y`. -/ @[simps] def binaryProductLimit (X Y : Type u) : IsLimit (binaryProductCone X Y) where lift (s : BinaryFan X Y) x := (s.fst x, s.snd x) fac _ j := Discrete.recOn j fun j => WalkingPair.casesOn j rfl rfl uniq _ _ w := funext fun x => Prod.ext (congr_fun (w ⟨left⟩) x) (congr_fun (w ⟨right⟩) x) #align category_theory.limits.types.binary_product_limit CategoryTheory.Limits.Types.binaryProductLimit /-- The category of types has `X × Y`, the usual cartesian product, as the binary product of `X` and `Y`. -/ @[simps] def binaryProductLimitCone (X Y : Type u) : Limits.LimitCone (pair X Y) := ⟨_, binaryProductLimit X Y⟩ #align category_theory.limits.types.binary_product_limit_cone CategoryTheory.Limits.Types.binaryProductLimitCone /-- The categorical binary product in `Type u` is cartesian product. -/ noncomputable def binaryProductIso (X Y : Type u) : Limits.prod X Y ≅ X × Y := limit.isoLimitCone (binaryProductLimitCone X Y) #align category_theory.limits.types.binary_product_iso CategoryTheory.Limits.Types.binaryProductIso @[elementwise (attr := simp)] theorem binaryProductIso_hom_comp_fst (X Y : Type u) : (binaryProductIso X Y).hom ≫ _root_.Prod.fst = Limits.prod.fst := limit.isoLimitCone_hom_π (binaryProductLimitCone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_product_iso_hom_comp_fst CategoryTheory.Limits.Types.binaryProductIso_hom_comp_fst @[elementwise (attr := simp)] theorem binaryProductIso_hom_comp_snd (X Y : Type u) : (binaryProductIso X Y).hom ≫ _root_.Prod.snd = Limits.prod.snd := limit.isoLimitCone_hom_π (binaryProductLimitCone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_product_iso_hom_comp_snd CategoryTheory.Limits.Types.binaryProductIso_hom_comp_snd @[elementwise (attr := simp)] theorem binaryProductIso_inv_comp_fst (X Y : Type u) : (binaryProductIso X Y).inv ≫ Limits.prod.fst = _root_.Prod.fst := limit.isoLimitCone_inv_π (binaryProductLimitCone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_product_iso_inv_comp_fst CategoryTheory.Limits.Types.binaryProductIso_inv_comp_fst @[elementwise (attr := simp)] theorem binaryProductIso_inv_comp_snd (X Y : Type u) : (binaryProductIso X Y).inv ≫ Limits.prod.snd = _root_.Prod.snd := limit.isoLimitCone_inv_π (binaryProductLimitCone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_product_iso_inv_comp_snd CategoryTheory.Limits.Types.binaryProductIso_inv_comp_snd -- porting note: it was originally @[simps (config := { typeMd := reducible })] -- We add the option `type_md` to tell `@[simps]` to not treat homomorphisms `X ⟶ Y` in `Type*` as -- a function type /-- The functor which sends `X, Y` to the product type `X × Y`. -/ @[simps] def binaryProductFunctor : Type u ⥤ Type u ⥤ Type u where obj X := { obj := fun Y => X × Y map := fun { Y₁ Y₂} f => (binaryProductLimit X Y₂).lift (BinaryFan.mk _root_.Prod.fst (_root_.Prod.snd ≫ f)) } map {X₁ X₂} f := { app := fun Y => (binaryProductLimit X₂ Y).lift (BinaryFan.mk (_root_.Prod.fst ≫ f) _root_.Prod.snd) } #align category_theory.limits.types.binary_product_functor CategoryTheory.Limits.Types.binaryProductFunctor /-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _) := by refine' NatIso.ofComponents (fun X => _) (fun _ => _) · refine' NatIso.ofComponents (fun Y => _) (fun _ => _) · exact ((limit.isLimit _).conePointUniqueUpToIso (binaryProductLimit X Y)).symm · apply Limits.prod.hom_ext <;> simp <;> rfl · ext : 2
apply Limits.prod.hom_ext
/-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _) := by refine' NatIso.ofComponents (fun X => _) (fun _ => _) · refine' NatIso.ofComponents (fun Y => _) (fun _ => _) · exact ((limit.isLimit _).conePointUniqueUpToIso (binaryProductLimit X Y)).symm · apply Limits.prod.hom_ext <;> simp <;> rfl · ext : 2
Mathlib.CategoryTheory.Limits.Shapes.Types.236_0.ctQAUYXLRXnvMGw
/-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _)
Mathlib_CategoryTheory_Limits_Shapes_Types
case refine'_2.w.h.h₁ X✝ Y✝ : Type u x✝¹ : X✝ ⟶ Y✝ x✝ : Type u ⊢ (binaryProductFunctor.map x✝¹ ≫ ((fun X => NatIso.ofComponents fun Y => (IsLimit.conePointUniqueUpToIso (limit.isLimit (pair X Y)) (binaryProductLimit X Y)).symm) Y✝).hom).app x✝ ≫ prod.fst = (((fun X => NatIso.ofComponents fun Y => (IsLimit.conePointUniqueUpToIso (limit.isLimit (pair X Y)) (binaryProductLimit X Y)).symm) X✝).hom ≫ prod.functor.map x✝¹).app x✝ ≫ prod.fst
/- Copyright (c) 2020 Scott Morrison. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Scott Morrison -/ import Mathlib.CategoryTheory.Limits.Types import Mathlib.CategoryTheory.Limits.Shapes.Products import Mathlib.CategoryTheory.Limits.Shapes.BinaryProducts import Mathlib.CategoryTheory.Limits.Shapes.Terminal import Mathlib.CategoryTheory.ConcreteCategory.Basic import Mathlib.Tactic.CategoryTheory.Elementwise #align_import category_theory.limits.shapes.types from "leanprover-community/mathlib"@"5dc6092d09e5e489106865241986f7f2ad28d4c8" /-! # Special shapes for limits in `Type`. The general shape (co)limits defined in `CategoryTheory.Limits.Types` are intended for use through the limits API, and the actual implementation should mostly be considered "sealed". In this file, we provide definitions of the "standard" special shapes of limits in `Type`, giving the expected definitional implementation: * the terminal object is `PUnit` * the binary product of `X` and `Y` is `X × Y` * the product of a family `f : J → Type` is `Π j, f j` * the coproduct of a family `f : J → Type` is `Σ j, f j` * the binary coproduct of `X` and `Y` is the sum type `X ⊕ Y` * the equalizer of a pair of maps `(g, h)` is the subtype `{x : Y // g x = h x}` * the coequalizer of a pair of maps `(f, g)` is the quotient of `Y` by `∀ x : Y, f x ~ g x` * the pullback of `f : X ⟶ Z` and `g : Y ⟶ Z` is the subtype `{ p : X × Y // f p.1 = g p.2 }` of the product We first construct terms of `IsLimit` and `LimitCone`, and then provide isomorphisms with the types generated by the `HasLimit` API. As an example, when setting up the monoidal category structure on `Type` we use the `Types.terminalLimitCone` and `Types.binaryProductLimitCone` definitions. -/ universe v u open CategoryTheory Limits namespace CategoryTheory.Limits.Types example : HasProducts.{v} (Type v) := inferInstance example [UnivLE.{v, u}] : HasProducts.{v} (Type u) := inferInstance -- This shortcut instance is required in `Mathlib.CategoryTheory.Closed.Types`, -- although I don't understand why, and wish it wasn't. instance : HasProducts.{v} (Type v) := inferInstance /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`. -/ @[simp 1001] theorem pi_lift_π_apply {β : Type v} [Small.{u} β] (f : β → Type u) {P : Type u} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := congr_fun (limit.lift_π (Fan.mk P s) ⟨b⟩) x #align category_theory.limits.types.pi_lift_π_apply CategoryTheory.Limits.Types.pi_lift_π_apply /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`, with specialized universes. -/ theorem pi_lift_π_apply' {β : Type v} (f : β → Type v) {P : Type v} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := by simp #align category_theory.limits.types.pi_lift_π_apply' CategoryTheory.Limits.Types.pi_lift_π_apply' /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`. -/ @[simp 1001] theorem pi_map_π_apply {β : Type v} [Small.{u} β] {f g : β → Type u} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := Limit.map_π_apply.{v, u} _ _ _ #align category_theory.limits.types.pi_map_π_apply CategoryTheory.Limits.Types.pi_map_π_apply /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`, with specialized universes. -/ theorem pi_map_π_apply' {β : Type v} {f g : β → Type v} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := by simp #align category_theory.limits.types.pi_map_π_apply' CategoryTheory.Limits.Types.pi_map_π_apply' /-- The category of types has `PUnit` as a terminal object. -/ def terminalLimitCone : Limits.LimitCone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cone := { pt := PUnit π := (Functor.uniqueFromEmpty _).hom } isLimit := { lift := fun _ _ => PUnit.unit fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext apply Subsingleton.elim } #align category_theory.limits.types.terminal_limit_cone CategoryTheory.Limits.Types.terminalLimitCone /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def terminalIso : ⊤_ Type u ≅ PUnit := limit.isoLimitCone terminalLimitCone.{u, 0} #align category_theory.limits.types.terminal_iso CategoryTheory.Limits.Types.terminalIso /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def isTerminalPunit : IsTerminal (PUnit : Type u) := terminalIsTerminal.ofIso terminalIso #align category_theory.limits.types.is_terminal_punit CategoryTheory.Limits.Types.isTerminalPunit -- porting note: the following three instances have been added to ease -- the automation in a definition in `AlgebraicTopology.SimplicialSet` noncomputable instance : Inhabited (⊤_ (Type u)) := ⟨@terminal.from (Type u) _ _ (ULift (Fin 1)) (ULift.up 0)⟩ instance : Subsingleton (⊤_ (Type u)) := ⟨fun a b => congr_fun (@Subsingleton.elim (_ ⟶ ⊤_ (Type u)) _ (fun _ => a) (fun _ => b)) (ULift.up (0 : Fin 1))⟩ noncomputable instance : Unique (⊤_ (Type u)) := Unique.mk' _ /-- A type is terminal if and only if it contains exactly one element. -/ noncomputable def isTerminalEquivUnique (X : Type u) : IsTerminal X ≃ Unique X := equivOfSubsingletonOfSubsingleton (fun h => ((Iso.toEquiv (terminalIsoIsTerminal h).symm).unique)) (fun _ => IsTerminal.ofIso terminalIsTerminal (Equiv.toIso (Equiv.equivOfUnique _ _))) /-- A type is terminal if and only if it is isomorphic to `PUnit`. -/ noncomputable def isTerminalEquivIsoPUnit (X : Type u) : IsTerminal X ≃ (X ≅ PUnit) := by calc IsTerminal X ≃ Unique X := isTerminalEquivUnique _ _ ≃ (X ≃ PUnit.{u + 1}) := uniqueEquivEquivUnique _ _ _ ≃ (X ≅ PUnit) := equivEquivIso /-- The category of types has `PEmpty` as an initial object. -/ def initialColimitCocone : Limits.ColimitCocone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cocone := { pt := PEmpty ι := (Functor.uniqueFromEmpty _).inv } isColimit := { desc := fun _ => by rintro ⟨⟩ fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext x; cases x } #align category_theory.limits.types.initial_colimit_cocone CategoryTheory.Limits.Types.initialColimitCocone /-- The initial object in `Type u` is `PEmpty`. -/ noncomputable def initialIso : ⊥_ Type u ≅ PEmpty := colimit.isoColimitCocone initialColimitCocone.{u, 0} #align category_theory.limits.types.initial_iso CategoryTheory.Limits.Types.initialIso /-- The initial object in `Type u` is `PEmpty`. -/ noncomputable def isInitialPunit : IsInitial (PEmpty : Type u) := initialIsInitial.ofIso initialIso #align category_theory.limits.types.is_initial_punit CategoryTheory.Limits.Types.isInitialPunit open CategoryTheory.Limits.WalkingPair -- We manually generate the other projection lemmas since the simp-normal form for the legs is -- otherwise not created correctly. /-- The product type `X × Y` forms a cone for the binary product of `X` and `Y`. -/ @[simps! pt] def binaryProductCone (X Y : Type u) : BinaryFan X Y := BinaryFan.mk _root_.Prod.fst _root_.Prod.snd #align category_theory.limits.types.binary_product_cone CategoryTheory.Limits.Types.binaryProductCone @[simp] theorem binaryProductCone_fst (X Y : Type u) : (binaryProductCone X Y).fst = _root_.Prod.fst := rfl #align category_theory.limits.types.binary_product_cone_fst CategoryTheory.Limits.Types.binaryProductCone_fst @[simp] theorem binaryProductCone_snd (X Y : Type u) : (binaryProductCone X Y).snd = _root_.Prod.snd := rfl #align category_theory.limits.types.binary_product_cone_snd CategoryTheory.Limits.Types.binaryProductCone_snd /-- The product type `X × Y` is a binary product for `X` and `Y`. -/ @[simps] def binaryProductLimit (X Y : Type u) : IsLimit (binaryProductCone X Y) where lift (s : BinaryFan X Y) x := (s.fst x, s.snd x) fac _ j := Discrete.recOn j fun j => WalkingPair.casesOn j rfl rfl uniq _ _ w := funext fun x => Prod.ext (congr_fun (w ⟨left⟩) x) (congr_fun (w ⟨right⟩) x) #align category_theory.limits.types.binary_product_limit CategoryTheory.Limits.Types.binaryProductLimit /-- The category of types has `X × Y`, the usual cartesian product, as the binary product of `X` and `Y`. -/ @[simps] def binaryProductLimitCone (X Y : Type u) : Limits.LimitCone (pair X Y) := ⟨_, binaryProductLimit X Y⟩ #align category_theory.limits.types.binary_product_limit_cone CategoryTheory.Limits.Types.binaryProductLimitCone /-- The categorical binary product in `Type u` is cartesian product. -/ noncomputable def binaryProductIso (X Y : Type u) : Limits.prod X Y ≅ X × Y := limit.isoLimitCone (binaryProductLimitCone X Y) #align category_theory.limits.types.binary_product_iso CategoryTheory.Limits.Types.binaryProductIso @[elementwise (attr := simp)] theorem binaryProductIso_hom_comp_fst (X Y : Type u) : (binaryProductIso X Y).hom ≫ _root_.Prod.fst = Limits.prod.fst := limit.isoLimitCone_hom_π (binaryProductLimitCone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_product_iso_hom_comp_fst CategoryTheory.Limits.Types.binaryProductIso_hom_comp_fst @[elementwise (attr := simp)] theorem binaryProductIso_hom_comp_snd (X Y : Type u) : (binaryProductIso X Y).hom ≫ _root_.Prod.snd = Limits.prod.snd := limit.isoLimitCone_hom_π (binaryProductLimitCone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_product_iso_hom_comp_snd CategoryTheory.Limits.Types.binaryProductIso_hom_comp_snd @[elementwise (attr := simp)] theorem binaryProductIso_inv_comp_fst (X Y : Type u) : (binaryProductIso X Y).inv ≫ Limits.prod.fst = _root_.Prod.fst := limit.isoLimitCone_inv_π (binaryProductLimitCone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_product_iso_inv_comp_fst CategoryTheory.Limits.Types.binaryProductIso_inv_comp_fst @[elementwise (attr := simp)] theorem binaryProductIso_inv_comp_snd (X Y : Type u) : (binaryProductIso X Y).inv ≫ Limits.prod.snd = _root_.Prod.snd := limit.isoLimitCone_inv_π (binaryProductLimitCone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_product_iso_inv_comp_snd CategoryTheory.Limits.Types.binaryProductIso_inv_comp_snd -- porting note: it was originally @[simps (config := { typeMd := reducible })] -- We add the option `type_md` to tell `@[simps]` to not treat homomorphisms `X ⟶ Y` in `Type*` as -- a function type /-- The functor which sends `X, Y` to the product type `X × Y`. -/ @[simps] def binaryProductFunctor : Type u ⥤ Type u ⥤ Type u where obj X := { obj := fun Y => X × Y map := fun { Y₁ Y₂} f => (binaryProductLimit X Y₂).lift (BinaryFan.mk _root_.Prod.fst (_root_.Prod.snd ≫ f)) } map {X₁ X₂} f := { app := fun Y => (binaryProductLimit X₂ Y).lift (BinaryFan.mk (_root_.Prod.fst ≫ f) _root_.Prod.snd) } #align category_theory.limits.types.binary_product_functor CategoryTheory.Limits.Types.binaryProductFunctor /-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _) := by refine' NatIso.ofComponents (fun X => _) (fun _ => _) · refine' NatIso.ofComponents (fun Y => _) (fun _ => _) · exact ((limit.isLimit _).conePointUniqueUpToIso (binaryProductLimit X Y)).symm · apply Limits.prod.hom_ext <;> simp <;> rfl · ext : 2 apply Limits.prod.hom_ext <;>
simp
/-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _) := by refine' NatIso.ofComponents (fun X => _) (fun _ => _) · refine' NatIso.ofComponents (fun Y => _) (fun _ => _) · exact ((limit.isLimit _).conePointUniqueUpToIso (binaryProductLimit X Y)).symm · apply Limits.prod.hom_ext <;> simp <;> rfl · ext : 2 apply Limits.prod.hom_ext <;>
Mathlib.CategoryTheory.Limits.Shapes.Types.236_0.ctQAUYXLRXnvMGw
/-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _)
Mathlib_CategoryTheory_Limits_Shapes_Types
case refine'_2.w.h.h₂ X✝ Y✝ : Type u x✝¹ : X✝ ⟶ Y✝ x✝ : Type u ⊢ (binaryProductFunctor.map x✝¹ ≫ ((fun X => NatIso.ofComponents fun Y => (IsLimit.conePointUniqueUpToIso (limit.isLimit (pair X Y)) (binaryProductLimit X Y)).symm) Y✝).hom).app x✝ ≫ prod.snd = (((fun X => NatIso.ofComponents fun Y => (IsLimit.conePointUniqueUpToIso (limit.isLimit (pair X Y)) (binaryProductLimit X Y)).symm) X✝).hom ≫ prod.functor.map x✝¹).app x✝ ≫ prod.snd
/- Copyright (c) 2020 Scott Morrison. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Scott Morrison -/ import Mathlib.CategoryTheory.Limits.Types import Mathlib.CategoryTheory.Limits.Shapes.Products import Mathlib.CategoryTheory.Limits.Shapes.BinaryProducts import Mathlib.CategoryTheory.Limits.Shapes.Terminal import Mathlib.CategoryTheory.ConcreteCategory.Basic import Mathlib.Tactic.CategoryTheory.Elementwise #align_import category_theory.limits.shapes.types from "leanprover-community/mathlib"@"5dc6092d09e5e489106865241986f7f2ad28d4c8" /-! # Special shapes for limits in `Type`. The general shape (co)limits defined in `CategoryTheory.Limits.Types` are intended for use through the limits API, and the actual implementation should mostly be considered "sealed". In this file, we provide definitions of the "standard" special shapes of limits in `Type`, giving the expected definitional implementation: * the terminal object is `PUnit` * the binary product of `X` and `Y` is `X × Y` * the product of a family `f : J → Type` is `Π j, f j` * the coproduct of a family `f : J → Type` is `Σ j, f j` * the binary coproduct of `X` and `Y` is the sum type `X ⊕ Y` * the equalizer of a pair of maps `(g, h)` is the subtype `{x : Y // g x = h x}` * the coequalizer of a pair of maps `(f, g)` is the quotient of `Y` by `∀ x : Y, f x ~ g x` * the pullback of `f : X ⟶ Z` and `g : Y ⟶ Z` is the subtype `{ p : X × Y // f p.1 = g p.2 }` of the product We first construct terms of `IsLimit` and `LimitCone`, and then provide isomorphisms with the types generated by the `HasLimit` API. As an example, when setting up the monoidal category structure on `Type` we use the `Types.terminalLimitCone` and `Types.binaryProductLimitCone` definitions. -/ universe v u open CategoryTheory Limits namespace CategoryTheory.Limits.Types example : HasProducts.{v} (Type v) := inferInstance example [UnivLE.{v, u}] : HasProducts.{v} (Type u) := inferInstance -- This shortcut instance is required in `Mathlib.CategoryTheory.Closed.Types`, -- although I don't understand why, and wish it wasn't. instance : HasProducts.{v} (Type v) := inferInstance /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`. -/ @[simp 1001] theorem pi_lift_π_apply {β : Type v} [Small.{u} β] (f : β → Type u) {P : Type u} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := congr_fun (limit.lift_π (Fan.mk P s) ⟨b⟩) x #align category_theory.limits.types.pi_lift_π_apply CategoryTheory.Limits.Types.pi_lift_π_apply /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`, with specialized universes. -/ theorem pi_lift_π_apply' {β : Type v} (f : β → Type v) {P : Type v} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := by simp #align category_theory.limits.types.pi_lift_π_apply' CategoryTheory.Limits.Types.pi_lift_π_apply' /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`. -/ @[simp 1001] theorem pi_map_π_apply {β : Type v} [Small.{u} β] {f g : β → Type u} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := Limit.map_π_apply.{v, u} _ _ _ #align category_theory.limits.types.pi_map_π_apply CategoryTheory.Limits.Types.pi_map_π_apply /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`, with specialized universes. -/ theorem pi_map_π_apply' {β : Type v} {f g : β → Type v} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := by simp #align category_theory.limits.types.pi_map_π_apply' CategoryTheory.Limits.Types.pi_map_π_apply' /-- The category of types has `PUnit` as a terminal object. -/ def terminalLimitCone : Limits.LimitCone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cone := { pt := PUnit π := (Functor.uniqueFromEmpty _).hom } isLimit := { lift := fun _ _ => PUnit.unit fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext apply Subsingleton.elim } #align category_theory.limits.types.terminal_limit_cone CategoryTheory.Limits.Types.terminalLimitCone /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def terminalIso : ⊤_ Type u ≅ PUnit := limit.isoLimitCone terminalLimitCone.{u, 0} #align category_theory.limits.types.terminal_iso CategoryTheory.Limits.Types.terminalIso /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def isTerminalPunit : IsTerminal (PUnit : Type u) := terminalIsTerminal.ofIso terminalIso #align category_theory.limits.types.is_terminal_punit CategoryTheory.Limits.Types.isTerminalPunit -- porting note: the following three instances have been added to ease -- the automation in a definition in `AlgebraicTopology.SimplicialSet` noncomputable instance : Inhabited (⊤_ (Type u)) := ⟨@terminal.from (Type u) _ _ (ULift (Fin 1)) (ULift.up 0)⟩ instance : Subsingleton (⊤_ (Type u)) := ⟨fun a b => congr_fun (@Subsingleton.elim (_ ⟶ ⊤_ (Type u)) _ (fun _ => a) (fun _ => b)) (ULift.up (0 : Fin 1))⟩ noncomputable instance : Unique (⊤_ (Type u)) := Unique.mk' _ /-- A type is terminal if and only if it contains exactly one element. -/ noncomputable def isTerminalEquivUnique (X : Type u) : IsTerminal X ≃ Unique X := equivOfSubsingletonOfSubsingleton (fun h => ((Iso.toEquiv (terminalIsoIsTerminal h).symm).unique)) (fun _ => IsTerminal.ofIso terminalIsTerminal (Equiv.toIso (Equiv.equivOfUnique _ _))) /-- A type is terminal if and only if it is isomorphic to `PUnit`. -/ noncomputable def isTerminalEquivIsoPUnit (X : Type u) : IsTerminal X ≃ (X ≅ PUnit) := by calc IsTerminal X ≃ Unique X := isTerminalEquivUnique _ _ ≃ (X ≃ PUnit.{u + 1}) := uniqueEquivEquivUnique _ _ _ ≃ (X ≅ PUnit) := equivEquivIso /-- The category of types has `PEmpty` as an initial object. -/ def initialColimitCocone : Limits.ColimitCocone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cocone := { pt := PEmpty ι := (Functor.uniqueFromEmpty _).inv } isColimit := { desc := fun _ => by rintro ⟨⟩ fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext x; cases x } #align category_theory.limits.types.initial_colimit_cocone CategoryTheory.Limits.Types.initialColimitCocone /-- The initial object in `Type u` is `PEmpty`. -/ noncomputable def initialIso : ⊥_ Type u ≅ PEmpty := colimit.isoColimitCocone initialColimitCocone.{u, 0} #align category_theory.limits.types.initial_iso CategoryTheory.Limits.Types.initialIso /-- The initial object in `Type u` is `PEmpty`. -/ noncomputable def isInitialPunit : IsInitial (PEmpty : Type u) := initialIsInitial.ofIso initialIso #align category_theory.limits.types.is_initial_punit CategoryTheory.Limits.Types.isInitialPunit open CategoryTheory.Limits.WalkingPair -- We manually generate the other projection lemmas since the simp-normal form for the legs is -- otherwise not created correctly. /-- The product type `X × Y` forms a cone for the binary product of `X` and `Y`. -/ @[simps! pt] def binaryProductCone (X Y : Type u) : BinaryFan X Y := BinaryFan.mk _root_.Prod.fst _root_.Prod.snd #align category_theory.limits.types.binary_product_cone CategoryTheory.Limits.Types.binaryProductCone @[simp] theorem binaryProductCone_fst (X Y : Type u) : (binaryProductCone X Y).fst = _root_.Prod.fst := rfl #align category_theory.limits.types.binary_product_cone_fst CategoryTheory.Limits.Types.binaryProductCone_fst @[simp] theorem binaryProductCone_snd (X Y : Type u) : (binaryProductCone X Y).snd = _root_.Prod.snd := rfl #align category_theory.limits.types.binary_product_cone_snd CategoryTheory.Limits.Types.binaryProductCone_snd /-- The product type `X × Y` is a binary product for `X` and `Y`. -/ @[simps] def binaryProductLimit (X Y : Type u) : IsLimit (binaryProductCone X Y) where lift (s : BinaryFan X Y) x := (s.fst x, s.snd x) fac _ j := Discrete.recOn j fun j => WalkingPair.casesOn j rfl rfl uniq _ _ w := funext fun x => Prod.ext (congr_fun (w ⟨left⟩) x) (congr_fun (w ⟨right⟩) x) #align category_theory.limits.types.binary_product_limit CategoryTheory.Limits.Types.binaryProductLimit /-- The category of types has `X × Y`, the usual cartesian product, as the binary product of `X` and `Y`. -/ @[simps] def binaryProductLimitCone (X Y : Type u) : Limits.LimitCone (pair X Y) := ⟨_, binaryProductLimit X Y⟩ #align category_theory.limits.types.binary_product_limit_cone CategoryTheory.Limits.Types.binaryProductLimitCone /-- The categorical binary product in `Type u` is cartesian product. -/ noncomputable def binaryProductIso (X Y : Type u) : Limits.prod X Y ≅ X × Y := limit.isoLimitCone (binaryProductLimitCone X Y) #align category_theory.limits.types.binary_product_iso CategoryTheory.Limits.Types.binaryProductIso @[elementwise (attr := simp)] theorem binaryProductIso_hom_comp_fst (X Y : Type u) : (binaryProductIso X Y).hom ≫ _root_.Prod.fst = Limits.prod.fst := limit.isoLimitCone_hom_π (binaryProductLimitCone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_product_iso_hom_comp_fst CategoryTheory.Limits.Types.binaryProductIso_hom_comp_fst @[elementwise (attr := simp)] theorem binaryProductIso_hom_comp_snd (X Y : Type u) : (binaryProductIso X Y).hom ≫ _root_.Prod.snd = Limits.prod.snd := limit.isoLimitCone_hom_π (binaryProductLimitCone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_product_iso_hom_comp_snd CategoryTheory.Limits.Types.binaryProductIso_hom_comp_snd @[elementwise (attr := simp)] theorem binaryProductIso_inv_comp_fst (X Y : Type u) : (binaryProductIso X Y).inv ≫ Limits.prod.fst = _root_.Prod.fst := limit.isoLimitCone_inv_π (binaryProductLimitCone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_product_iso_inv_comp_fst CategoryTheory.Limits.Types.binaryProductIso_inv_comp_fst @[elementwise (attr := simp)] theorem binaryProductIso_inv_comp_snd (X Y : Type u) : (binaryProductIso X Y).inv ≫ Limits.prod.snd = _root_.Prod.snd := limit.isoLimitCone_inv_π (binaryProductLimitCone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_product_iso_inv_comp_snd CategoryTheory.Limits.Types.binaryProductIso_inv_comp_snd -- porting note: it was originally @[simps (config := { typeMd := reducible })] -- We add the option `type_md` to tell `@[simps]` to not treat homomorphisms `X ⟶ Y` in `Type*` as -- a function type /-- The functor which sends `X, Y` to the product type `X × Y`. -/ @[simps] def binaryProductFunctor : Type u ⥤ Type u ⥤ Type u where obj X := { obj := fun Y => X × Y map := fun { Y₁ Y₂} f => (binaryProductLimit X Y₂).lift (BinaryFan.mk _root_.Prod.fst (_root_.Prod.snd ≫ f)) } map {X₁ X₂} f := { app := fun Y => (binaryProductLimit X₂ Y).lift (BinaryFan.mk (_root_.Prod.fst ≫ f) _root_.Prod.snd) } #align category_theory.limits.types.binary_product_functor CategoryTheory.Limits.Types.binaryProductFunctor /-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _) := by refine' NatIso.ofComponents (fun X => _) (fun _ => _) · refine' NatIso.ofComponents (fun Y => _) (fun _ => _) · exact ((limit.isLimit _).conePointUniqueUpToIso (binaryProductLimit X Y)).symm · apply Limits.prod.hom_ext <;> simp <;> rfl · ext : 2 apply Limits.prod.hom_ext <;>
simp
/-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _) := by refine' NatIso.ofComponents (fun X => _) (fun _ => _) · refine' NatIso.ofComponents (fun Y => _) (fun _ => _) · exact ((limit.isLimit _).conePointUniqueUpToIso (binaryProductLimit X Y)).symm · apply Limits.prod.hom_ext <;> simp <;> rfl · ext : 2 apply Limits.prod.hom_ext <;>
Mathlib.CategoryTheory.Limits.Shapes.Types.236_0.ctQAUYXLRXnvMGw
/-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _)
Mathlib_CategoryTheory_Limits_Shapes_Types
case refine'_2.w.h.h₁ X✝ Y✝ : Type u x✝¹ : X✝ ⟶ Y✝ x✝ : Type u ⊢ (binaryProductFunctor.map x✝¹).app x✝ ≫ _root_.Prod.fst = _root_.Prod.fst ≫ x✝¹
/- Copyright (c) 2020 Scott Morrison. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Scott Morrison -/ import Mathlib.CategoryTheory.Limits.Types import Mathlib.CategoryTheory.Limits.Shapes.Products import Mathlib.CategoryTheory.Limits.Shapes.BinaryProducts import Mathlib.CategoryTheory.Limits.Shapes.Terminal import Mathlib.CategoryTheory.ConcreteCategory.Basic import Mathlib.Tactic.CategoryTheory.Elementwise #align_import category_theory.limits.shapes.types from "leanprover-community/mathlib"@"5dc6092d09e5e489106865241986f7f2ad28d4c8" /-! # Special shapes for limits in `Type`. The general shape (co)limits defined in `CategoryTheory.Limits.Types` are intended for use through the limits API, and the actual implementation should mostly be considered "sealed". In this file, we provide definitions of the "standard" special shapes of limits in `Type`, giving the expected definitional implementation: * the terminal object is `PUnit` * the binary product of `X` and `Y` is `X × Y` * the product of a family `f : J → Type` is `Π j, f j` * the coproduct of a family `f : J → Type` is `Σ j, f j` * the binary coproduct of `X` and `Y` is the sum type `X ⊕ Y` * the equalizer of a pair of maps `(g, h)` is the subtype `{x : Y // g x = h x}` * the coequalizer of a pair of maps `(f, g)` is the quotient of `Y` by `∀ x : Y, f x ~ g x` * the pullback of `f : X ⟶ Z` and `g : Y ⟶ Z` is the subtype `{ p : X × Y // f p.1 = g p.2 }` of the product We first construct terms of `IsLimit` and `LimitCone`, and then provide isomorphisms with the types generated by the `HasLimit` API. As an example, when setting up the monoidal category structure on `Type` we use the `Types.terminalLimitCone` and `Types.binaryProductLimitCone` definitions. -/ universe v u open CategoryTheory Limits namespace CategoryTheory.Limits.Types example : HasProducts.{v} (Type v) := inferInstance example [UnivLE.{v, u}] : HasProducts.{v} (Type u) := inferInstance -- This shortcut instance is required in `Mathlib.CategoryTheory.Closed.Types`, -- although I don't understand why, and wish it wasn't. instance : HasProducts.{v} (Type v) := inferInstance /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`. -/ @[simp 1001] theorem pi_lift_π_apply {β : Type v} [Small.{u} β] (f : β → Type u) {P : Type u} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := congr_fun (limit.lift_π (Fan.mk P s) ⟨b⟩) x #align category_theory.limits.types.pi_lift_π_apply CategoryTheory.Limits.Types.pi_lift_π_apply /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`, with specialized universes. -/ theorem pi_lift_π_apply' {β : Type v} (f : β → Type v) {P : Type v} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := by simp #align category_theory.limits.types.pi_lift_π_apply' CategoryTheory.Limits.Types.pi_lift_π_apply' /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`. -/ @[simp 1001] theorem pi_map_π_apply {β : Type v} [Small.{u} β] {f g : β → Type u} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := Limit.map_π_apply.{v, u} _ _ _ #align category_theory.limits.types.pi_map_π_apply CategoryTheory.Limits.Types.pi_map_π_apply /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`, with specialized universes. -/ theorem pi_map_π_apply' {β : Type v} {f g : β → Type v} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := by simp #align category_theory.limits.types.pi_map_π_apply' CategoryTheory.Limits.Types.pi_map_π_apply' /-- The category of types has `PUnit` as a terminal object. -/ def terminalLimitCone : Limits.LimitCone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cone := { pt := PUnit π := (Functor.uniqueFromEmpty _).hom } isLimit := { lift := fun _ _ => PUnit.unit fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext apply Subsingleton.elim } #align category_theory.limits.types.terminal_limit_cone CategoryTheory.Limits.Types.terminalLimitCone /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def terminalIso : ⊤_ Type u ≅ PUnit := limit.isoLimitCone terminalLimitCone.{u, 0} #align category_theory.limits.types.terminal_iso CategoryTheory.Limits.Types.terminalIso /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def isTerminalPunit : IsTerminal (PUnit : Type u) := terminalIsTerminal.ofIso terminalIso #align category_theory.limits.types.is_terminal_punit CategoryTheory.Limits.Types.isTerminalPunit -- porting note: the following three instances have been added to ease -- the automation in a definition in `AlgebraicTopology.SimplicialSet` noncomputable instance : Inhabited (⊤_ (Type u)) := ⟨@terminal.from (Type u) _ _ (ULift (Fin 1)) (ULift.up 0)⟩ instance : Subsingleton (⊤_ (Type u)) := ⟨fun a b => congr_fun (@Subsingleton.elim (_ ⟶ ⊤_ (Type u)) _ (fun _ => a) (fun _ => b)) (ULift.up (0 : Fin 1))⟩ noncomputable instance : Unique (⊤_ (Type u)) := Unique.mk' _ /-- A type is terminal if and only if it contains exactly one element. -/ noncomputable def isTerminalEquivUnique (X : Type u) : IsTerminal X ≃ Unique X := equivOfSubsingletonOfSubsingleton (fun h => ((Iso.toEquiv (terminalIsoIsTerminal h).symm).unique)) (fun _ => IsTerminal.ofIso terminalIsTerminal (Equiv.toIso (Equiv.equivOfUnique _ _))) /-- A type is terminal if and only if it is isomorphic to `PUnit`. -/ noncomputable def isTerminalEquivIsoPUnit (X : Type u) : IsTerminal X ≃ (X ≅ PUnit) := by calc IsTerminal X ≃ Unique X := isTerminalEquivUnique _ _ ≃ (X ≃ PUnit.{u + 1}) := uniqueEquivEquivUnique _ _ _ ≃ (X ≅ PUnit) := equivEquivIso /-- The category of types has `PEmpty` as an initial object. -/ def initialColimitCocone : Limits.ColimitCocone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cocone := { pt := PEmpty ι := (Functor.uniqueFromEmpty _).inv } isColimit := { desc := fun _ => by rintro ⟨⟩ fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext x; cases x } #align category_theory.limits.types.initial_colimit_cocone CategoryTheory.Limits.Types.initialColimitCocone /-- The initial object in `Type u` is `PEmpty`. -/ noncomputable def initialIso : ⊥_ Type u ≅ PEmpty := colimit.isoColimitCocone initialColimitCocone.{u, 0} #align category_theory.limits.types.initial_iso CategoryTheory.Limits.Types.initialIso /-- The initial object in `Type u` is `PEmpty`. -/ noncomputable def isInitialPunit : IsInitial (PEmpty : Type u) := initialIsInitial.ofIso initialIso #align category_theory.limits.types.is_initial_punit CategoryTheory.Limits.Types.isInitialPunit open CategoryTheory.Limits.WalkingPair -- We manually generate the other projection lemmas since the simp-normal form for the legs is -- otherwise not created correctly. /-- The product type `X × Y` forms a cone for the binary product of `X` and `Y`. -/ @[simps! pt] def binaryProductCone (X Y : Type u) : BinaryFan X Y := BinaryFan.mk _root_.Prod.fst _root_.Prod.snd #align category_theory.limits.types.binary_product_cone CategoryTheory.Limits.Types.binaryProductCone @[simp] theorem binaryProductCone_fst (X Y : Type u) : (binaryProductCone X Y).fst = _root_.Prod.fst := rfl #align category_theory.limits.types.binary_product_cone_fst CategoryTheory.Limits.Types.binaryProductCone_fst @[simp] theorem binaryProductCone_snd (X Y : Type u) : (binaryProductCone X Y).snd = _root_.Prod.snd := rfl #align category_theory.limits.types.binary_product_cone_snd CategoryTheory.Limits.Types.binaryProductCone_snd /-- The product type `X × Y` is a binary product for `X` and `Y`. -/ @[simps] def binaryProductLimit (X Y : Type u) : IsLimit (binaryProductCone X Y) where lift (s : BinaryFan X Y) x := (s.fst x, s.snd x) fac _ j := Discrete.recOn j fun j => WalkingPair.casesOn j rfl rfl uniq _ _ w := funext fun x => Prod.ext (congr_fun (w ⟨left⟩) x) (congr_fun (w ⟨right⟩) x) #align category_theory.limits.types.binary_product_limit CategoryTheory.Limits.Types.binaryProductLimit /-- The category of types has `X × Y`, the usual cartesian product, as the binary product of `X` and `Y`. -/ @[simps] def binaryProductLimitCone (X Y : Type u) : Limits.LimitCone (pair X Y) := ⟨_, binaryProductLimit X Y⟩ #align category_theory.limits.types.binary_product_limit_cone CategoryTheory.Limits.Types.binaryProductLimitCone /-- The categorical binary product in `Type u` is cartesian product. -/ noncomputable def binaryProductIso (X Y : Type u) : Limits.prod X Y ≅ X × Y := limit.isoLimitCone (binaryProductLimitCone X Y) #align category_theory.limits.types.binary_product_iso CategoryTheory.Limits.Types.binaryProductIso @[elementwise (attr := simp)] theorem binaryProductIso_hom_comp_fst (X Y : Type u) : (binaryProductIso X Y).hom ≫ _root_.Prod.fst = Limits.prod.fst := limit.isoLimitCone_hom_π (binaryProductLimitCone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_product_iso_hom_comp_fst CategoryTheory.Limits.Types.binaryProductIso_hom_comp_fst @[elementwise (attr := simp)] theorem binaryProductIso_hom_comp_snd (X Y : Type u) : (binaryProductIso X Y).hom ≫ _root_.Prod.snd = Limits.prod.snd := limit.isoLimitCone_hom_π (binaryProductLimitCone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_product_iso_hom_comp_snd CategoryTheory.Limits.Types.binaryProductIso_hom_comp_snd @[elementwise (attr := simp)] theorem binaryProductIso_inv_comp_fst (X Y : Type u) : (binaryProductIso X Y).inv ≫ Limits.prod.fst = _root_.Prod.fst := limit.isoLimitCone_inv_π (binaryProductLimitCone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_product_iso_inv_comp_fst CategoryTheory.Limits.Types.binaryProductIso_inv_comp_fst @[elementwise (attr := simp)] theorem binaryProductIso_inv_comp_snd (X Y : Type u) : (binaryProductIso X Y).inv ≫ Limits.prod.snd = _root_.Prod.snd := limit.isoLimitCone_inv_π (binaryProductLimitCone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_product_iso_inv_comp_snd CategoryTheory.Limits.Types.binaryProductIso_inv_comp_snd -- porting note: it was originally @[simps (config := { typeMd := reducible })] -- We add the option `type_md` to tell `@[simps]` to not treat homomorphisms `X ⟶ Y` in `Type*` as -- a function type /-- The functor which sends `X, Y` to the product type `X × Y`. -/ @[simps] def binaryProductFunctor : Type u ⥤ Type u ⥤ Type u where obj X := { obj := fun Y => X × Y map := fun { Y₁ Y₂} f => (binaryProductLimit X Y₂).lift (BinaryFan.mk _root_.Prod.fst (_root_.Prod.snd ≫ f)) } map {X₁ X₂} f := { app := fun Y => (binaryProductLimit X₂ Y).lift (BinaryFan.mk (_root_.Prod.fst ≫ f) _root_.Prod.snd) } #align category_theory.limits.types.binary_product_functor CategoryTheory.Limits.Types.binaryProductFunctor /-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _) := by refine' NatIso.ofComponents (fun X => _) (fun _ => _) · refine' NatIso.ofComponents (fun Y => _) (fun _ => _) · exact ((limit.isLimit _).conePointUniqueUpToIso (binaryProductLimit X Y)).symm · apply Limits.prod.hom_ext <;> simp <;> rfl · ext : 2 apply Limits.prod.hom_ext <;> simp <;>
rfl
/-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _) := by refine' NatIso.ofComponents (fun X => _) (fun _ => _) · refine' NatIso.ofComponents (fun Y => _) (fun _ => _) · exact ((limit.isLimit _).conePointUniqueUpToIso (binaryProductLimit X Y)).symm · apply Limits.prod.hom_ext <;> simp <;> rfl · ext : 2 apply Limits.prod.hom_ext <;> simp <;>
Mathlib.CategoryTheory.Limits.Shapes.Types.236_0.ctQAUYXLRXnvMGw
/-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _)
Mathlib_CategoryTheory_Limits_Shapes_Types
case refine'_2.w.h.h₂ X✝ Y✝ : Type u x✝¹ : X✝ ⟶ Y✝ x✝ : Type u ⊢ (binaryProductFunctor.map x✝¹).app x✝ ≫ _root_.Prod.snd = _root_.Prod.snd
/- Copyright (c) 2020 Scott Morrison. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Scott Morrison -/ import Mathlib.CategoryTheory.Limits.Types import Mathlib.CategoryTheory.Limits.Shapes.Products import Mathlib.CategoryTheory.Limits.Shapes.BinaryProducts import Mathlib.CategoryTheory.Limits.Shapes.Terminal import Mathlib.CategoryTheory.ConcreteCategory.Basic import Mathlib.Tactic.CategoryTheory.Elementwise #align_import category_theory.limits.shapes.types from "leanprover-community/mathlib"@"5dc6092d09e5e489106865241986f7f2ad28d4c8" /-! # Special shapes for limits in `Type`. The general shape (co)limits defined in `CategoryTheory.Limits.Types` are intended for use through the limits API, and the actual implementation should mostly be considered "sealed". In this file, we provide definitions of the "standard" special shapes of limits in `Type`, giving the expected definitional implementation: * the terminal object is `PUnit` * the binary product of `X` and `Y` is `X × Y` * the product of a family `f : J → Type` is `Π j, f j` * the coproduct of a family `f : J → Type` is `Σ j, f j` * the binary coproduct of `X` and `Y` is the sum type `X ⊕ Y` * the equalizer of a pair of maps `(g, h)` is the subtype `{x : Y // g x = h x}` * the coequalizer of a pair of maps `(f, g)` is the quotient of `Y` by `∀ x : Y, f x ~ g x` * the pullback of `f : X ⟶ Z` and `g : Y ⟶ Z` is the subtype `{ p : X × Y // f p.1 = g p.2 }` of the product We first construct terms of `IsLimit` and `LimitCone`, and then provide isomorphisms with the types generated by the `HasLimit` API. As an example, when setting up the monoidal category structure on `Type` we use the `Types.terminalLimitCone` and `Types.binaryProductLimitCone` definitions. -/ universe v u open CategoryTheory Limits namespace CategoryTheory.Limits.Types example : HasProducts.{v} (Type v) := inferInstance example [UnivLE.{v, u}] : HasProducts.{v} (Type u) := inferInstance -- This shortcut instance is required in `Mathlib.CategoryTheory.Closed.Types`, -- although I don't understand why, and wish it wasn't. instance : HasProducts.{v} (Type v) := inferInstance /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`. -/ @[simp 1001] theorem pi_lift_π_apply {β : Type v} [Small.{u} β] (f : β → Type u) {P : Type u} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := congr_fun (limit.lift_π (Fan.mk P s) ⟨b⟩) x #align category_theory.limits.types.pi_lift_π_apply CategoryTheory.Limits.Types.pi_lift_π_apply /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`, with specialized universes. -/ theorem pi_lift_π_apply' {β : Type v} (f : β → Type v) {P : Type v} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := by simp #align category_theory.limits.types.pi_lift_π_apply' CategoryTheory.Limits.Types.pi_lift_π_apply' /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`. -/ @[simp 1001] theorem pi_map_π_apply {β : Type v} [Small.{u} β] {f g : β → Type u} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := Limit.map_π_apply.{v, u} _ _ _ #align category_theory.limits.types.pi_map_π_apply CategoryTheory.Limits.Types.pi_map_π_apply /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`, with specialized universes. -/ theorem pi_map_π_apply' {β : Type v} {f g : β → Type v} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := by simp #align category_theory.limits.types.pi_map_π_apply' CategoryTheory.Limits.Types.pi_map_π_apply' /-- The category of types has `PUnit` as a terminal object. -/ def terminalLimitCone : Limits.LimitCone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cone := { pt := PUnit π := (Functor.uniqueFromEmpty _).hom } isLimit := { lift := fun _ _ => PUnit.unit fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext apply Subsingleton.elim } #align category_theory.limits.types.terminal_limit_cone CategoryTheory.Limits.Types.terminalLimitCone /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def terminalIso : ⊤_ Type u ≅ PUnit := limit.isoLimitCone terminalLimitCone.{u, 0} #align category_theory.limits.types.terminal_iso CategoryTheory.Limits.Types.terminalIso /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def isTerminalPunit : IsTerminal (PUnit : Type u) := terminalIsTerminal.ofIso terminalIso #align category_theory.limits.types.is_terminal_punit CategoryTheory.Limits.Types.isTerminalPunit -- porting note: the following three instances have been added to ease -- the automation in a definition in `AlgebraicTopology.SimplicialSet` noncomputable instance : Inhabited (⊤_ (Type u)) := ⟨@terminal.from (Type u) _ _ (ULift (Fin 1)) (ULift.up 0)⟩ instance : Subsingleton (⊤_ (Type u)) := ⟨fun a b => congr_fun (@Subsingleton.elim (_ ⟶ ⊤_ (Type u)) _ (fun _ => a) (fun _ => b)) (ULift.up (0 : Fin 1))⟩ noncomputable instance : Unique (⊤_ (Type u)) := Unique.mk' _ /-- A type is terminal if and only if it contains exactly one element. -/ noncomputable def isTerminalEquivUnique (X : Type u) : IsTerminal X ≃ Unique X := equivOfSubsingletonOfSubsingleton (fun h => ((Iso.toEquiv (terminalIsoIsTerminal h).symm).unique)) (fun _ => IsTerminal.ofIso terminalIsTerminal (Equiv.toIso (Equiv.equivOfUnique _ _))) /-- A type is terminal if and only if it is isomorphic to `PUnit`. -/ noncomputable def isTerminalEquivIsoPUnit (X : Type u) : IsTerminal X ≃ (X ≅ PUnit) := by calc IsTerminal X ≃ Unique X := isTerminalEquivUnique _ _ ≃ (X ≃ PUnit.{u + 1}) := uniqueEquivEquivUnique _ _ _ ≃ (X ≅ PUnit) := equivEquivIso /-- The category of types has `PEmpty` as an initial object. -/ def initialColimitCocone : Limits.ColimitCocone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cocone := { pt := PEmpty ι := (Functor.uniqueFromEmpty _).inv } isColimit := { desc := fun _ => by rintro ⟨⟩ fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext x; cases x } #align category_theory.limits.types.initial_colimit_cocone CategoryTheory.Limits.Types.initialColimitCocone /-- The initial object in `Type u` is `PEmpty`. -/ noncomputable def initialIso : ⊥_ Type u ≅ PEmpty := colimit.isoColimitCocone initialColimitCocone.{u, 0} #align category_theory.limits.types.initial_iso CategoryTheory.Limits.Types.initialIso /-- The initial object in `Type u` is `PEmpty`. -/ noncomputable def isInitialPunit : IsInitial (PEmpty : Type u) := initialIsInitial.ofIso initialIso #align category_theory.limits.types.is_initial_punit CategoryTheory.Limits.Types.isInitialPunit open CategoryTheory.Limits.WalkingPair -- We manually generate the other projection lemmas since the simp-normal form for the legs is -- otherwise not created correctly. /-- The product type `X × Y` forms a cone for the binary product of `X` and `Y`. -/ @[simps! pt] def binaryProductCone (X Y : Type u) : BinaryFan X Y := BinaryFan.mk _root_.Prod.fst _root_.Prod.snd #align category_theory.limits.types.binary_product_cone CategoryTheory.Limits.Types.binaryProductCone @[simp] theorem binaryProductCone_fst (X Y : Type u) : (binaryProductCone X Y).fst = _root_.Prod.fst := rfl #align category_theory.limits.types.binary_product_cone_fst CategoryTheory.Limits.Types.binaryProductCone_fst @[simp] theorem binaryProductCone_snd (X Y : Type u) : (binaryProductCone X Y).snd = _root_.Prod.snd := rfl #align category_theory.limits.types.binary_product_cone_snd CategoryTheory.Limits.Types.binaryProductCone_snd /-- The product type `X × Y` is a binary product for `X` and `Y`. -/ @[simps] def binaryProductLimit (X Y : Type u) : IsLimit (binaryProductCone X Y) where lift (s : BinaryFan X Y) x := (s.fst x, s.snd x) fac _ j := Discrete.recOn j fun j => WalkingPair.casesOn j rfl rfl uniq _ _ w := funext fun x => Prod.ext (congr_fun (w ⟨left⟩) x) (congr_fun (w ⟨right⟩) x) #align category_theory.limits.types.binary_product_limit CategoryTheory.Limits.Types.binaryProductLimit /-- The category of types has `X × Y`, the usual cartesian product, as the binary product of `X` and `Y`. -/ @[simps] def binaryProductLimitCone (X Y : Type u) : Limits.LimitCone (pair X Y) := ⟨_, binaryProductLimit X Y⟩ #align category_theory.limits.types.binary_product_limit_cone CategoryTheory.Limits.Types.binaryProductLimitCone /-- The categorical binary product in `Type u` is cartesian product. -/ noncomputable def binaryProductIso (X Y : Type u) : Limits.prod X Y ≅ X × Y := limit.isoLimitCone (binaryProductLimitCone X Y) #align category_theory.limits.types.binary_product_iso CategoryTheory.Limits.Types.binaryProductIso @[elementwise (attr := simp)] theorem binaryProductIso_hom_comp_fst (X Y : Type u) : (binaryProductIso X Y).hom ≫ _root_.Prod.fst = Limits.prod.fst := limit.isoLimitCone_hom_π (binaryProductLimitCone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_product_iso_hom_comp_fst CategoryTheory.Limits.Types.binaryProductIso_hom_comp_fst @[elementwise (attr := simp)] theorem binaryProductIso_hom_comp_snd (X Y : Type u) : (binaryProductIso X Y).hom ≫ _root_.Prod.snd = Limits.prod.snd := limit.isoLimitCone_hom_π (binaryProductLimitCone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_product_iso_hom_comp_snd CategoryTheory.Limits.Types.binaryProductIso_hom_comp_snd @[elementwise (attr := simp)] theorem binaryProductIso_inv_comp_fst (X Y : Type u) : (binaryProductIso X Y).inv ≫ Limits.prod.fst = _root_.Prod.fst := limit.isoLimitCone_inv_π (binaryProductLimitCone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_product_iso_inv_comp_fst CategoryTheory.Limits.Types.binaryProductIso_inv_comp_fst @[elementwise (attr := simp)] theorem binaryProductIso_inv_comp_snd (X Y : Type u) : (binaryProductIso X Y).inv ≫ Limits.prod.snd = _root_.Prod.snd := limit.isoLimitCone_inv_π (binaryProductLimitCone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_product_iso_inv_comp_snd CategoryTheory.Limits.Types.binaryProductIso_inv_comp_snd -- porting note: it was originally @[simps (config := { typeMd := reducible })] -- We add the option `type_md` to tell `@[simps]` to not treat homomorphisms `X ⟶ Y` in `Type*` as -- a function type /-- The functor which sends `X, Y` to the product type `X × Y`. -/ @[simps] def binaryProductFunctor : Type u ⥤ Type u ⥤ Type u where obj X := { obj := fun Y => X × Y map := fun { Y₁ Y₂} f => (binaryProductLimit X Y₂).lift (BinaryFan.mk _root_.Prod.fst (_root_.Prod.snd ≫ f)) } map {X₁ X₂} f := { app := fun Y => (binaryProductLimit X₂ Y).lift (BinaryFan.mk (_root_.Prod.fst ≫ f) _root_.Prod.snd) } #align category_theory.limits.types.binary_product_functor CategoryTheory.Limits.Types.binaryProductFunctor /-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _) := by refine' NatIso.ofComponents (fun X => _) (fun _ => _) · refine' NatIso.ofComponents (fun Y => _) (fun _ => _) · exact ((limit.isLimit _).conePointUniqueUpToIso (binaryProductLimit X Y)).symm · apply Limits.prod.hom_ext <;> simp <;> rfl · ext : 2 apply Limits.prod.hom_ext <;> simp <;>
rfl
/-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _) := by refine' NatIso.ofComponents (fun X => _) (fun _ => _) · refine' NatIso.ofComponents (fun Y => _) (fun _ => _) · exact ((limit.isLimit _).conePointUniqueUpToIso (binaryProductLimit X Y)).symm · apply Limits.prod.hom_ext <;> simp <;> rfl · ext : 2 apply Limits.prod.hom_ext <;> simp <;>
Mathlib.CategoryTheory.Limits.Shapes.Types.236_0.ctQAUYXLRXnvMGw
/-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _)
Mathlib_CategoryTheory_Limits_Shapes_Types
X Y : Type u c : BinaryCofan X Y ⊢ Nonempty (IsColimit c) ↔ Injective (BinaryCofan.inl c) ∧ Injective (BinaryCofan.inr c) ∧ IsCompl (Set.range (BinaryCofan.inl c)) (Set.range (BinaryCofan.inr c))
/- Copyright (c) 2020 Scott Morrison. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Scott Morrison -/ import Mathlib.CategoryTheory.Limits.Types import Mathlib.CategoryTheory.Limits.Shapes.Products import Mathlib.CategoryTheory.Limits.Shapes.BinaryProducts import Mathlib.CategoryTheory.Limits.Shapes.Terminal import Mathlib.CategoryTheory.ConcreteCategory.Basic import Mathlib.Tactic.CategoryTheory.Elementwise #align_import category_theory.limits.shapes.types from "leanprover-community/mathlib"@"5dc6092d09e5e489106865241986f7f2ad28d4c8" /-! # Special shapes for limits in `Type`. The general shape (co)limits defined in `CategoryTheory.Limits.Types` are intended for use through the limits API, and the actual implementation should mostly be considered "sealed". In this file, we provide definitions of the "standard" special shapes of limits in `Type`, giving the expected definitional implementation: * the terminal object is `PUnit` * the binary product of `X` and `Y` is `X × Y` * the product of a family `f : J → Type` is `Π j, f j` * the coproduct of a family `f : J → Type` is `Σ j, f j` * the binary coproduct of `X` and `Y` is the sum type `X ⊕ Y` * the equalizer of a pair of maps `(g, h)` is the subtype `{x : Y // g x = h x}` * the coequalizer of a pair of maps `(f, g)` is the quotient of `Y` by `∀ x : Y, f x ~ g x` * the pullback of `f : X ⟶ Z` and `g : Y ⟶ Z` is the subtype `{ p : X × Y // f p.1 = g p.2 }` of the product We first construct terms of `IsLimit` and `LimitCone`, and then provide isomorphisms with the types generated by the `HasLimit` API. As an example, when setting up the monoidal category structure on `Type` we use the `Types.terminalLimitCone` and `Types.binaryProductLimitCone` definitions. -/ universe v u open CategoryTheory Limits namespace CategoryTheory.Limits.Types example : HasProducts.{v} (Type v) := inferInstance example [UnivLE.{v, u}] : HasProducts.{v} (Type u) := inferInstance -- This shortcut instance is required in `Mathlib.CategoryTheory.Closed.Types`, -- although I don't understand why, and wish it wasn't. instance : HasProducts.{v} (Type v) := inferInstance /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`. -/ @[simp 1001] theorem pi_lift_π_apply {β : Type v} [Small.{u} β] (f : β → Type u) {P : Type u} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := congr_fun (limit.lift_π (Fan.mk P s) ⟨b⟩) x #align category_theory.limits.types.pi_lift_π_apply CategoryTheory.Limits.Types.pi_lift_π_apply /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`, with specialized universes. -/ theorem pi_lift_π_apply' {β : Type v} (f : β → Type v) {P : Type v} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := by simp #align category_theory.limits.types.pi_lift_π_apply' CategoryTheory.Limits.Types.pi_lift_π_apply' /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`. -/ @[simp 1001] theorem pi_map_π_apply {β : Type v} [Small.{u} β] {f g : β → Type u} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := Limit.map_π_apply.{v, u} _ _ _ #align category_theory.limits.types.pi_map_π_apply CategoryTheory.Limits.Types.pi_map_π_apply /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`, with specialized universes. -/ theorem pi_map_π_apply' {β : Type v} {f g : β → Type v} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := by simp #align category_theory.limits.types.pi_map_π_apply' CategoryTheory.Limits.Types.pi_map_π_apply' /-- The category of types has `PUnit` as a terminal object. -/ def terminalLimitCone : Limits.LimitCone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cone := { pt := PUnit π := (Functor.uniqueFromEmpty _).hom } isLimit := { lift := fun _ _ => PUnit.unit fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext apply Subsingleton.elim } #align category_theory.limits.types.terminal_limit_cone CategoryTheory.Limits.Types.terminalLimitCone /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def terminalIso : ⊤_ Type u ≅ PUnit := limit.isoLimitCone terminalLimitCone.{u, 0} #align category_theory.limits.types.terminal_iso CategoryTheory.Limits.Types.terminalIso /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def isTerminalPunit : IsTerminal (PUnit : Type u) := terminalIsTerminal.ofIso terminalIso #align category_theory.limits.types.is_terminal_punit CategoryTheory.Limits.Types.isTerminalPunit -- porting note: the following three instances have been added to ease -- the automation in a definition in `AlgebraicTopology.SimplicialSet` noncomputable instance : Inhabited (⊤_ (Type u)) := ⟨@terminal.from (Type u) _ _ (ULift (Fin 1)) (ULift.up 0)⟩ instance : Subsingleton (⊤_ (Type u)) := ⟨fun a b => congr_fun (@Subsingleton.elim (_ ⟶ ⊤_ (Type u)) _ (fun _ => a) (fun _ => b)) (ULift.up (0 : Fin 1))⟩ noncomputable instance : Unique (⊤_ (Type u)) := Unique.mk' _ /-- A type is terminal if and only if it contains exactly one element. -/ noncomputable def isTerminalEquivUnique (X : Type u) : IsTerminal X ≃ Unique X := equivOfSubsingletonOfSubsingleton (fun h => ((Iso.toEquiv (terminalIsoIsTerminal h).symm).unique)) (fun _ => IsTerminal.ofIso terminalIsTerminal (Equiv.toIso (Equiv.equivOfUnique _ _))) /-- A type is terminal if and only if it is isomorphic to `PUnit`. -/ noncomputable def isTerminalEquivIsoPUnit (X : Type u) : IsTerminal X ≃ (X ≅ PUnit) := by calc IsTerminal X ≃ Unique X := isTerminalEquivUnique _ _ ≃ (X ≃ PUnit.{u + 1}) := uniqueEquivEquivUnique _ _ _ ≃ (X ≅ PUnit) := equivEquivIso /-- The category of types has `PEmpty` as an initial object. -/ def initialColimitCocone : Limits.ColimitCocone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cocone := { pt := PEmpty ι := (Functor.uniqueFromEmpty _).inv } isColimit := { desc := fun _ => by rintro ⟨⟩ fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext x; cases x } #align category_theory.limits.types.initial_colimit_cocone CategoryTheory.Limits.Types.initialColimitCocone /-- The initial object in `Type u` is `PEmpty`. -/ noncomputable def initialIso : ⊥_ Type u ≅ PEmpty := colimit.isoColimitCocone initialColimitCocone.{u, 0} #align category_theory.limits.types.initial_iso CategoryTheory.Limits.Types.initialIso /-- The initial object in `Type u` is `PEmpty`. -/ noncomputable def isInitialPunit : IsInitial (PEmpty : Type u) := initialIsInitial.ofIso initialIso #align category_theory.limits.types.is_initial_punit CategoryTheory.Limits.Types.isInitialPunit open CategoryTheory.Limits.WalkingPair -- We manually generate the other projection lemmas since the simp-normal form for the legs is -- otherwise not created correctly. /-- The product type `X × Y` forms a cone for the binary product of `X` and `Y`. -/ @[simps! pt] def binaryProductCone (X Y : Type u) : BinaryFan X Y := BinaryFan.mk _root_.Prod.fst _root_.Prod.snd #align category_theory.limits.types.binary_product_cone CategoryTheory.Limits.Types.binaryProductCone @[simp] theorem binaryProductCone_fst (X Y : Type u) : (binaryProductCone X Y).fst = _root_.Prod.fst := rfl #align category_theory.limits.types.binary_product_cone_fst CategoryTheory.Limits.Types.binaryProductCone_fst @[simp] theorem binaryProductCone_snd (X Y : Type u) : (binaryProductCone X Y).snd = _root_.Prod.snd := rfl #align category_theory.limits.types.binary_product_cone_snd CategoryTheory.Limits.Types.binaryProductCone_snd /-- The product type `X × Y` is a binary product for `X` and `Y`. -/ @[simps] def binaryProductLimit (X Y : Type u) : IsLimit (binaryProductCone X Y) where lift (s : BinaryFan X Y) x := (s.fst x, s.snd x) fac _ j := Discrete.recOn j fun j => WalkingPair.casesOn j rfl rfl uniq _ _ w := funext fun x => Prod.ext (congr_fun (w ⟨left⟩) x) (congr_fun (w ⟨right⟩) x) #align category_theory.limits.types.binary_product_limit CategoryTheory.Limits.Types.binaryProductLimit /-- The category of types has `X × Y`, the usual cartesian product, as the binary product of `X` and `Y`. -/ @[simps] def binaryProductLimitCone (X Y : Type u) : Limits.LimitCone (pair X Y) := ⟨_, binaryProductLimit X Y⟩ #align category_theory.limits.types.binary_product_limit_cone CategoryTheory.Limits.Types.binaryProductLimitCone /-- The categorical binary product in `Type u` is cartesian product. -/ noncomputable def binaryProductIso (X Y : Type u) : Limits.prod X Y ≅ X × Y := limit.isoLimitCone (binaryProductLimitCone X Y) #align category_theory.limits.types.binary_product_iso CategoryTheory.Limits.Types.binaryProductIso @[elementwise (attr := simp)] theorem binaryProductIso_hom_comp_fst (X Y : Type u) : (binaryProductIso X Y).hom ≫ _root_.Prod.fst = Limits.prod.fst := limit.isoLimitCone_hom_π (binaryProductLimitCone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_product_iso_hom_comp_fst CategoryTheory.Limits.Types.binaryProductIso_hom_comp_fst @[elementwise (attr := simp)] theorem binaryProductIso_hom_comp_snd (X Y : Type u) : (binaryProductIso X Y).hom ≫ _root_.Prod.snd = Limits.prod.snd := limit.isoLimitCone_hom_π (binaryProductLimitCone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_product_iso_hom_comp_snd CategoryTheory.Limits.Types.binaryProductIso_hom_comp_snd @[elementwise (attr := simp)] theorem binaryProductIso_inv_comp_fst (X Y : Type u) : (binaryProductIso X Y).inv ≫ Limits.prod.fst = _root_.Prod.fst := limit.isoLimitCone_inv_π (binaryProductLimitCone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_product_iso_inv_comp_fst CategoryTheory.Limits.Types.binaryProductIso_inv_comp_fst @[elementwise (attr := simp)] theorem binaryProductIso_inv_comp_snd (X Y : Type u) : (binaryProductIso X Y).inv ≫ Limits.prod.snd = _root_.Prod.snd := limit.isoLimitCone_inv_π (binaryProductLimitCone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_product_iso_inv_comp_snd CategoryTheory.Limits.Types.binaryProductIso_inv_comp_snd -- porting note: it was originally @[simps (config := { typeMd := reducible })] -- We add the option `type_md` to tell `@[simps]` to not treat homomorphisms `X ⟶ Y` in `Type*` as -- a function type /-- The functor which sends `X, Y` to the product type `X × Y`. -/ @[simps] def binaryProductFunctor : Type u ⥤ Type u ⥤ Type u where obj X := { obj := fun Y => X × Y map := fun { Y₁ Y₂} f => (binaryProductLimit X Y₂).lift (BinaryFan.mk _root_.Prod.fst (_root_.Prod.snd ≫ f)) } map {X₁ X₂} f := { app := fun Y => (binaryProductLimit X₂ Y).lift (BinaryFan.mk (_root_.Prod.fst ≫ f) _root_.Prod.snd) } #align category_theory.limits.types.binary_product_functor CategoryTheory.Limits.Types.binaryProductFunctor /-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _) := by refine' NatIso.ofComponents (fun X => _) (fun _ => _) · refine' NatIso.ofComponents (fun Y => _) (fun _ => _) · exact ((limit.isLimit _).conePointUniqueUpToIso (binaryProductLimit X Y)).symm · apply Limits.prod.hom_ext <;> simp <;> rfl · ext : 2 apply Limits.prod.hom_ext <;> simp <;> rfl #align category_theory.limits.types.binary_product_iso_prod CategoryTheory.Limits.Types.binaryProductIsoProd /-- The sum type `X ⊕ Y` forms a cocone for the binary coproduct of `X` and `Y`. -/ @[simps!] def binaryCoproductCocone (X Y : Type u) : Cocone (pair X Y) := BinaryCofan.mk Sum.inl Sum.inr #align category_theory.limits.types.binary_coproduct_cocone CategoryTheory.Limits.Types.binaryCoproductCocone /-- The sum type `X ⊕ Y` is a binary coproduct for `X` and `Y`. -/ @[simps] def binaryCoproductColimit (X Y : Type u) : IsColimit (binaryCoproductCocone X Y) where desc := fun s : BinaryCofan X Y => Sum.elim s.inl s.inr fac _ j := Discrete.recOn j fun j => WalkingPair.casesOn j rfl rfl uniq _ _ w := funext fun x => Sum.casesOn x (congr_fun (w ⟨left⟩)) (congr_fun (w ⟨right⟩)) #align category_theory.limits.types.binary_coproduct_colimit CategoryTheory.Limits.Types.binaryCoproductColimit /-- The category of types has `X ⊕ Y`, as the binary coproduct of `X` and `Y`. -/ def binaryCoproductColimitCocone (X Y : Type u) : Limits.ColimitCocone (pair X Y) := ⟨_, binaryCoproductColimit X Y⟩ #align category_theory.limits.types.binary_coproduct_colimit_cocone CategoryTheory.Limits.Types.binaryCoproductColimitCocone /-- The categorical binary coproduct in `Type u` is the sum `X ⊕ Y`. -/ noncomputable def binaryCoproductIso (X Y : Type u) : Limits.coprod X Y ≅ Sum X Y := colimit.isoColimitCocone (binaryCoproductColimitCocone X Y) #align category_theory.limits.types.binary_coproduct_iso CategoryTheory.Limits.Types.binaryCoproductIso --open CategoryTheory.Type @[elementwise (attr := simp)] theorem binaryCoproductIso_inl_comp_hom (X Y : Type u) : Limits.coprod.inl ≫ (binaryCoproductIso X Y).hom = Sum.inl := colimit.isoColimitCocone_ι_hom (binaryCoproductColimitCocone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_coproduct_iso_inl_comp_hom CategoryTheory.Limits.Types.binaryCoproductIso_inl_comp_hom @[elementwise (attr := simp)] theorem binaryCoproductIso_inr_comp_hom (X Y : Type u) : Limits.coprod.inr ≫ (binaryCoproductIso X Y).hom = Sum.inr := colimit.isoColimitCocone_ι_hom (binaryCoproductColimitCocone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_coproduct_iso_inr_comp_hom CategoryTheory.Limits.Types.binaryCoproductIso_inr_comp_hom @[elementwise (attr := simp)] theorem binaryCoproductIso_inl_comp_inv (X Y : Type u) : ↾(Sum.inl : X ⟶ Sum X Y) ≫ (binaryCoproductIso X Y).inv = Limits.coprod.inl := colimit.isoColimitCocone_ι_inv (binaryCoproductColimitCocone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_coproduct_iso_inl_comp_inv CategoryTheory.Limits.Types.binaryCoproductIso_inl_comp_inv @[elementwise (attr := simp)] theorem binaryCoproductIso_inr_comp_inv (X Y : Type u) : ↾(Sum.inr : Y ⟶ Sum X Y) ≫ (binaryCoproductIso X Y).inv = Limits.coprod.inr := colimit.isoColimitCocone_ι_inv (binaryCoproductColimitCocone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_coproduct_iso_inr_comp_inv CategoryTheory.Limits.Types.binaryCoproductIso_inr_comp_inv open Function (Injective) theorem binaryCofan_isColimit_iff {X Y : Type u} (c : BinaryCofan X Y) : Nonempty (IsColimit c) ↔ Injective c.inl ∧ Injective c.inr ∧ IsCompl (Set.range c.inl) (Set.range c.inr) := by
classical constructor · rintro ⟨h⟩ rw [← show _ = c.inl from h.comp_coconePointUniqueUpToIso_inv (binaryCoproductColimit X Y) ⟨WalkingPair.left⟩, ← show _ = c.inr from h.comp_coconePointUniqueUpToIso_inv (binaryCoproductColimit X Y) ⟨WalkingPair.right⟩] dsimp [binaryCoproductCocone] refine' ⟨(h.coconePointUniqueUpToIso (binaryCoproductColimit X Y)).symm.toEquiv.injective.comp Sum.inl_injective, (h.coconePointUniqueUpToIso (binaryCoproductColimit X Y)).symm.toEquiv.injective.comp Sum.inr_injective, _⟩ erw [Set.range_comp, ← eq_compl_iff_isCompl, Set.range_comp _ Sum.inr, ← Set.image_compl_eq (h.coconePointUniqueUpToIso (binaryCoproductColimit X Y)).symm.toEquiv.bijective] simp · rintro ⟨h₁, h₂, h₃⟩ have : ∀ x, x ∈ Set.range c.inl ∨ x ∈ Set.range c.inr := by rw [eq_compl_iff_isCompl.mpr h₃.symm] exact fun _ => or_not refine' ⟨BinaryCofan.IsColimit.mk _ _ _ _ _⟩ · intro T f g x exact if h : x ∈ Set.range c.inl then f ((Equiv.ofInjective _ h₁).symm ⟨x, h⟩) else g ((Equiv.ofInjective _ h₂).symm ⟨x, (this x).resolve_left h⟩) · intro T f g funext x dsimp simp [h₁.eq_iff] · intro T f g funext x dsimp simp only [Set.mem_range, Equiv.ofInjective_symm_apply, dite_eq_right_iff, forall_exists_index] intro y e have : c.inr x ∈ Set.range c.inl ⊓ Set.range c.inr := ⟨⟨_, e⟩, ⟨_, rfl⟩⟩ rw [disjoint_iff.mp h₃.1] at this exact this.elim · rintro T _ _ m rfl rfl funext x dsimp split_ifs <;> exact congr_arg _ (Equiv.apply_ofInjective_symm _ ⟨_, _⟩).symm
theorem binaryCofan_isColimit_iff {X Y : Type u} (c : BinaryCofan X Y) : Nonempty (IsColimit c) ↔ Injective c.inl ∧ Injective c.inr ∧ IsCompl (Set.range c.inl) (Set.range c.inr) := by
Mathlib.CategoryTheory.Limits.Shapes.Types.302_0.ctQAUYXLRXnvMGw
theorem binaryCofan_isColimit_iff {X Y : Type u} (c : BinaryCofan X Y) : Nonempty (IsColimit c) ↔ Injective c.inl ∧ Injective c.inr ∧ IsCompl (Set.range c.inl) (Set.range c.inr)
Mathlib_CategoryTheory_Limits_Shapes_Types
X Y : Type u c : BinaryCofan X Y ⊢ Nonempty (IsColimit c) ↔ Injective (BinaryCofan.inl c) ∧ Injective (BinaryCofan.inr c) ∧ IsCompl (Set.range (BinaryCofan.inl c)) (Set.range (BinaryCofan.inr c))
/- Copyright (c) 2020 Scott Morrison. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Scott Morrison -/ import Mathlib.CategoryTheory.Limits.Types import Mathlib.CategoryTheory.Limits.Shapes.Products import Mathlib.CategoryTheory.Limits.Shapes.BinaryProducts import Mathlib.CategoryTheory.Limits.Shapes.Terminal import Mathlib.CategoryTheory.ConcreteCategory.Basic import Mathlib.Tactic.CategoryTheory.Elementwise #align_import category_theory.limits.shapes.types from "leanprover-community/mathlib"@"5dc6092d09e5e489106865241986f7f2ad28d4c8" /-! # Special shapes for limits in `Type`. The general shape (co)limits defined in `CategoryTheory.Limits.Types` are intended for use through the limits API, and the actual implementation should mostly be considered "sealed". In this file, we provide definitions of the "standard" special shapes of limits in `Type`, giving the expected definitional implementation: * the terminal object is `PUnit` * the binary product of `X` and `Y` is `X × Y` * the product of a family `f : J → Type` is `Π j, f j` * the coproduct of a family `f : J → Type` is `Σ j, f j` * the binary coproduct of `X` and `Y` is the sum type `X ⊕ Y` * the equalizer of a pair of maps `(g, h)` is the subtype `{x : Y // g x = h x}` * the coequalizer of a pair of maps `(f, g)` is the quotient of `Y` by `∀ x : Y, f x ~ g x` * the pullback of `f : X ⟶ Z` and `g : Y ⟶ Z` is the subtype `{ p : X × Y // f p.1 = g p.2 }` of the product We first construct terms of `IsLimit` and `LimitCone`, and then provide isomorphisms with the types generated by the `HasLimit` API. As an example, when setting up the monoidal category structure on `Type` we use the `Types.terminalLimitCone` and `Types.binaryProductLimitCone` definitions. -/ universe v u open CategoryTheory Limits namespace CategoryTheory.Limits.Types example : HasProducts.{v} (Type v) := inferInstance example [UnivLE.{v, u}] : HasProducts.{v} (Type u) := inferInstance -- This shortcut instance is required in `Mathlib.CategoryTheory.Closed.Types`, -- although I don't understand why, and wish it wasn't. instance : HasProducts.{v} (Type v) := inferInstance /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`. -/ @[simp 1001] theorem pi_lift_π_apply {β : Type v} [Small.{u} β] (f : β → Type u) {P : Type u} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := congr_fun (limit.lift_π (Fan.mk P s) ⟨b⟩) x #align category_theory.limits.types.pi_lift_π_apply CategoryTheory.Limits.Types.pi_lift_π_apply /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`, with specialized universes. -/ theorem pi_lift_π_apply' {β : Type v} (f : β → Type v) {P : Type v} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := by simp #align category_theory.limits.types.pi_lift_π_apply' CategoryTheory.Limits.Types.pi_lift_π_apply' /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`. -/ @[simp 1001] theorem pi_map_π_apply {β : Type v} [Small.{u} β] {f g : β → Type u} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := Limit.map_π_apply.{v, u} _ _ _ #align category_theory.limits.types.pi_map_π_apply CategoryTheory.Limits.Types.pi_map_π_apply /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`, with specialized universes. -/ theorem pi_map_π_apply' {β : Type v} {f g : β → Type v} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := by simp #align category_theory.limits.types.pi_map_π_apply' CategoryTheory.Limits.Types.pi_map_π_apply' /-- The category of types has `PUnit` as a terminal object. -/ def terminalLimitCone : Limits.LimitCone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cone := { pt := PUnit π := (Functor.uniqueFromEmpty _).hom } isLimit := { lift := fun _ _ => PUnit.unit fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext apply Subsingleton.elim } #align category_theory.limits.types.terminal_limit_cone CategoryTheory.Limits.Types.terminalLimitCone /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def terminalIso : ⊤_ Type u ≅ PUnit := limit.isoLimitCone terminalLimitCone.{u, 0} #align category_theory.limits.types.terminal_iso CategoryTheory.Limits.Types.terminalIso /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def isTerminalPunit : IsTerminal (PUnit : Type u) := terminalIsTerminal.ofIso terminalIso #align category_theory.limits.types.is_terminal_punit CategoryTheory.Limits.Types.isTerminalPunit -- porting note: the following three instances have been added to ease -- the automation in a definition in `AlgebraicTopology.SimplicialSet` noncomputable instance : Inhabited (⊤_ (Type u)) := ⟨@terminal.from (Type u) _ _ (ULift (Fin 1)) (ULift.up 0)⟩ instance : Subsingleton (⊤_ (Type u)) := ⟨fun a b => congr_fun (@Subsingleton.elim (_ ⟶ ⊤_ (Type u)) _ (fun _ => a) (fun _ => b)) (ULift.up (0 : Fin 1))⟩ noncomputable instance : Unique (⊤_ (Type u)) := Unique.mk' _ /-- A type is terminal if and only if it contains exactly one element. -/ noncomputable def isTerminalEquivUnique (X : Type u) : IsTerminal X ≃ Unique X := equivOfSubsingletonOfSubsingleton (fun h => ((Iso.toEquiv (terminalIsoIsTerminal h).symm).unique)) (fun _ => IsTerminal.ofIso terminalIsTerminal (Equiv.toIso (Equiv.equivOfUnique _ _))) /-- A type is terminal if and only if it is isomorphic to `PUnit`. -/ noncomputable def isTerminalEquivIsoPUnit (X : Type u) : IsTerminal X ≃ (X ≅ PUnit) := by calc IsTerminal X ≃ Unique X := isTerminalEquivUnique _ _ ≃ (X ≃ PUnit.{u + 1}) := uniqueEquivEquivUnique _ _ _ ≃ (X ≅ PUnit) := equivEquivIso /-- The category of types has `PEmpty` as an initial object. -/ def initialColimitCocone : Limits.ColimitCocone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cocone := { pt := PEmpty ι := (Functor.uniqueFromEmpty _).inv } isColimit := { desc := fun _ => by rintro ⟨⟩ fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext x; cases x } #align category_theory.limits.types.initial_colimit_cocone CategoryTheory.Limits.Types.initialColimitCocone /-- The initial object in `Type u` is `PEmpty`. -/ noncomputable def initialIso : ⊥_ Type u ≅ PEmpty := colimit.isoColimitCocone initialColimitCocone.{u, 0} #align category_theory.limits.types.initial_iso CategoryTheory.Limits.Types.initialIso /-- The initial object in `Type u` is `PEmpty`. -/ noncomputable def isInitialPunit : IsInitial (PEmpty : Type u) := initialIsInitial.ofIso initialIso #align category_theory.limits.types.is_initial_punit CategoryTheory.Limits.Types.isInitialPunit open CategoryTheory.Limits.WalkingPair -- We manually generate the other projection lemmas since the simp-normal form for the legs is -- otherwise not created correctly. /-- The product type `X × Y` forms a cone for the binary product of `X` and `Y`. -/ @[simps! pt] def binaryProductCone (X Y : Type u) : BinaryFan X Y := BinaryFan.mk _root_.Prod.fst _root_.Prod.snd #align category_theory.limits.types.binary_product_cone CategoryTheory.Limits.Types.binaryProductCone @[simp] theorem binaryProductCone_fst (X Y : Type u) : (binaryProductCone X Y).fst = _root_.Prod.fst := rfl #align category_theory.limits.types.binary_product_cone_fst CategoryTheory.Limits.Types.binaryProductCone_fst @[simp] theorem binaryProductCone_snd (X Y : Type u) : (binaryProductCone X Y).snd = _root_.Prod.snd := rfl #align category_theory.limits.types.binary_product_cone_snd CategoryTheory.Limits.Types.binaryProductCone_snd /-- The product type `X × Y` is a binary product for `X` and `Y`. -/ @[simps] def binaryProductLimit (X Y : Type u) : IsLimit (binaryProductCone X Y) where lift (s : BinaryFan X Y) x := (s.fst x, s.snd x) fac _ j := Discrete.recOn j fun j => WalkingPair.casesOn j rfl rfl uniq _ _ w := funext fun x => Prod.ext (congr_fun (w ⟨left⟩) x) (congr_fun (w ⟨right⟩) x) #align category_theory.limits.types.binary_product_limit CategoryTheory.Limits.Types.binaryProductLimit /-- The category of types has `X × Y`, the usual cartesian product, as the binary product of `X` and `Y`. -/ @[simps] def binaryProductLimitCone (X Y : Type u) : Limits.LimitCone (pair X Y) := ⟨_, binaryProductLimit X Y⟩ #align category_theory.limits.types.binary_product_limit_cone CategoryTheory.Limits.Types.binaryProductLimitCone /-- The categorical binary product in `Type u` is cartesian product. -/ noncomputable def binaryProductIso (X Y : Type u) : Limits.prod X Y ≅ X × Y := limit.isoLimitCone (binaryProductLimitCone X Y) #align category_theory.limits.types.binary_product_iso CategoryTheory.Limits.Types.binaryProductIso @[elementwise (attr := simp)] theorem binaryProductIso_hom_comp_fst (X Y : Type u) : (binaryProductIso X Y).hom ≫ _root_.Prod.fst = Limits.prod.fst := limit.isoLimitCone_hom_π (binaryProductLimitCone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_product_iso_hom_comp_fst CategoryTheory.Limits.Types.binaryProductIso_hom_comp_fst @[elementwise (attr := simp)] theorem binaryProductIso_hom_comp_snd (X Y : Type u) : (binaryProductIso X Y).hom ≫ _root_.Prod.snd = Limits.prod.snd := limit.isoLimitCone_hom_π (binaryProductLimitCone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_product_iso_hom_comp_snd CategoryTheory.Limits.Types.binaryProductIso_hom_comp_snd @[elementwise (attr := simp)] theorem binaryProductIso_inv_comp_fst (X Y : Type u) : (binaryProductIso X Y).inv ≫ Limits.prod.fst = _root_.Prod.fst := limit.isoLimitCone_inv_π (binaryProductLimitCone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_product_iso_inv_comp_fst CategoryTheory.Limits.Types.binaryProductIso_inv_comp_fst @[elementwise (attr := simp)] theorem binaryProductIso_inv_comp_snd (X Y : Type u) : (binaryProductIso X Y).inv ≫ Limits.prod.snd = _root_.Prod.snd := limit.isoLimitCone_inv_π (binaryProductLimitCone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_product_iso_inv_comp_snd CategoryTheory.Limits.Types.binaryProductIso_inv_comp_snd -- porting note: it was originally @[simps (config := { typeMd := reducible })] -- We add the option `type_md` to tell `@[simps]` to not treat homomorphisms `X ⟶ Y` in `Type*` as -- a function type /-- The functor which sends `X, Y` to the product type `X × Y`. -/ @[simps] def binaryProductFunctor : Type u ⥤ Type u ⥤ Type u where obj X := { obj := fun Y => X × Y map := fun { Y₁ Y₂} f => (binaryProductLimit X Y₂).lift (BinaryFan.mk _root_.Prod.fst (_root_.Prod.snd ≫ f)) } map {X₁ X₂} f := { app := fun Y => (binaryProductLimit X₂ Y).lift (BinaryFan.mk (_root_.Prod.fst ≫ f) _root_.Prod.snd) } #align category_theory.limits.types.binary_product_functor CategoryTheory.Limits.Types.binaryProductFunctor /-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _) := by refine' NatIso.ofComponents (fun X => _) (fun _ => _) · refine' NatIso.ofComponents (fun Y => _) (fun _ => _) · exact ((limit.isLimit _).conePointUniqueUpToIso (binaryProductLimit X Y)).symm · apply Limits.prod.hom_ext <;> simp <;> rfl · ext : 2 apply Limits.prod.hom_ext <;> simp <;> rfl #align category_theory.limits.types.binary_product_iso_prod CategoryTheory.Limits.Types.binaryProductIsoProd /-- The sum type `X ⊕ Y` forms a cocone for the binary coproduct of `X` and `Y`. -/ @[simps!] def binaryCoproductCocone (X Y : Type u) : Cocone (pair X Y) := BinaryCofan.mk Sum.inl Sum.inr #align category_theory.limits.types.binary_coproduct_cocone CategoryTheory.Limits.Types.binaryCoproductCocone /-- The sum type `X ⊕ Y` is a binary coproduct for `X` and `Y`. -/ @[simps] def binaryCoproductColimit (X Y : Type u) : IsColimit (binaryCoproductCocone X Y) where desc := fun s : BinaryCofan X Y => Sum.elim s.inl s.inr fac _ j := Discrete.recOn j fun j => WalkingPair.casesOn j rfl rfl uniq _ _ w := funext fun x => Sum.casesOn x (congr_fun (w ⟨left⟩)) (congr_fun (w ⟨right⟩)) #align category_theory.limits.types.binary_coproduct_colimit CategoryTheory.Limits.Types.binaryCoproductColimit /-- The category of types has `X ⊕ Y`, as the binary coproduct of `X` and `Y`. -/ def binaryCoproductColimitCocone (X Y : Type u) : Limits.ColimitCocone (pair X Y) := ⟨_, binaryCoproductColimit X Y⟩ #align category_theory.limits.types.binary_coproduct_colimit_cocone CategoryTheory.Limits.Types.binaryCoproductColimitCocone /-- The categorical binary coproduct in `Type u` is the sum `X ⊕ Y`. -/ noncomputable def binaryCoproductIso (X Y : Type u) : Limits.coprod X Y ≅ Sum X Y := colimit.isoColimitCocone (binaryCoproductColimitCocone X Y) #align category_theory.limits.types.binary_coproduct_iso CategoryTheory.Limits.Types.binaryCoproductIso --open CategoryTheory.Type @[elementwise (attr := simp)] theorem binaryCoproductIso_inl_comp_hom (X Y : Type u) : Limits.coprod.inl ≫ (binaryCoproductIso X Y).hom = Sum.inl := colimit.isoColimitCocone_ι_hom (binaryCoproductColimitCocone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_coproduct_iso_inl_comp_hom CategoryTheory.Limits.Types.binaryCoproductIso_inl_comp_hom @[elementwise (attr := simp)] theorem binaryCoproductIso_inr_comp_hom (X Y : Type u) : Limits.coprod.inr ≫ (binaryCoproductIso X Y).hom = Sum.inr := colimit.isoColimitCocone_ι_hom (binaryCoproductColimitCocone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_coproduct_iso_inr_comp_hom CategoryTheory.Limits.Types.binaryCoproductIso_inr_comp_hom @[elementwise (attr := simp)] theorem binaryCoproductIso_inl_comp_inv (X Y : Type u) : ↾(Sum.inl : X ⟶ Sum X Y) ≫ (binaryCoproductIso X Y).inv = Limits.coprod.inl := colimit.isoColimitCocone_ι_inv (binaryCoproductColimitCocone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_coproduct_iso_inl_comp_inv CategoryTheory.Limits.Types.binaryCoproductIso_inl_comp_inv @[elementwise (attr := simp)] theorem binaryCoproductIso_inr_comp_inv (X Y : Type u) : ↾(Sum.inr : Y ⟶ Sum X Y) ≫ (binaryCoproductIso X Y).inv = Limits.coprod.inr := colimit.isoColimitCocone_ι_inv (binaryCoproductColimitCocone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_coproduct_iso_inr_comp_inv CategoryTheory.Limits.Types.binaryCoproductIso_inr_comp_inv open Function (Injective) theorem binaryCofan_isColimit_iff {X Y : Type u} (c : BinaryCofan X Y) : Nonempty (IsColimit c) ↔ Injective c.inl ∧ Injective c.inr ∧ IsCompl (Set.range c.inl) (Set.range c.inr) := by classical
constructor
theorem binaryCofan_isColimit_iff {X Y : Type u} (c : BinaryCofan X Y) : Nonempty (IsColimit c) ↔ Injective c.inl ∧ Injective c.inr ∧ IsCompl (Set.range c.inl) (Set.range c.inr) := by classical
Mathlib.CategoryTheory.Limits.Shapes.Types.302_0.ctQAUYXLRXnvMGw
theorem binaryCofan_isColimit_iff {X Y : Type u} (c : BinaryCofan X Y) : Nonempty (IsColimit c) ↔ Injective c.inl ∧ Injective c.inr ∧ IsCompl (Set.range c.inl) (Set.range c.inr)
Mathlib_CategoryTheory_Limits_Shapes_Types
case mp X Y : Type u c : BinaryCofan X Y ⊢ Nonempty (IsColimit c) → Injective (BinaryCofan.inl c) ∧ Injective (BinaryCofan.inr c) ∧ IsCompl (Set.range (BinaryCofan.inl c)) (Set.range (BinaryCofan.inr c))
/- Copyright (c) 2020 Scott Morrison. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Scott Morrison -/ import Mathlib.CategoryTheory.Limits.Types import Mathlib.CategoryTheory.Limits.Shapes.Products import Mathlib.CategoryTheory.Limits.Shapes.BinaryProducts import Mathlib.CategoryTheory.Limits.Shapes.Terminal import Mathlib.CategoryTheory.ConcreteCategory.Basic import Mathlib.Tactic.CategoryTheory.Elementwise #align_import category_theory.limits.shapes.types from "leanprover-community/mathlib"@"5dc6092d09e5e489106865241986f7f2ad28d4c8" /-! # Special shapes for limits in `Type`. The general shape (co)limits defined in `CategoryTheory.Limits.Types` are intended for use through the limits API, and the actual implementation should mostly be considered "sealed". In this file, we provide definitions of the "standard" special shapes of limits in `Type`, giving the expected definitional implementation: * the terminal object is `PUnit` * the binary product of `X` and `Y` is `X × Y` * the product of a family `f : J → Type` is `Π j, f j` * the coproduct of a family `f : J → Type` is `Σ j, f j` * the binary coproduct of `X` and `Y` is the sum type `X ⊕ Y` * the equalizer of a pair of maps `(g, h)` is the subtype `{x : Y // g x = h x}` * the coequalizer of a pair of maps `(f, g)` is the quotient of `Y` by `∀ x : Y, f x ~ g x` * the pullback of `f : X ⟶ Z` and `g : Y ⟶ Z` is the subtype `{ p : X × Y // f p.1 = g p.2 }` of the product We first construct terms of `IsLimit` and `LimitCone`, and then provide isomorphisms with the types generated by the `HasLimit` API. As an example, when setting up the monoidal category structure on `Type` we use the `Types.terminalLimitCone` and `Types.binaryProductLimitCone` definitions. -/ universe v u open CategoryTheory Limits namespace CategoryTheory.Limits.Types example : HasProducts.{v} (Type v) := inferInstance example [UnivLE.{v, u}] : HasProducts.{v} (Type u) := inferInstance -- This shortcut instance is required in `Mathlib.CategoryTheory.Closed.Types`, -- although I don't understand why, and wish it wasn't. instance : HasProducts.{v} (Type v) := inferInstance /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`. -/ @[simp 1001] theorem pi_lift_π_apply {β : Type v} [Small.{u} β] (f : β → Type u) {P : Type u} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := congr_fun (limit.lift_π (Fan.mk P s) ⟨b⟩) x #align category_theory.limits.types.pi_lift_π_apply CategoryTheory.Limits.Types.pi_lift_π_apply /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`, with specialized universes. -/ theorem pi_lift_π_apply' {β : Type v} (f : β → Type v) {P : Type v} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := by simp #align category_theory.limits.types.pi_lift_π_apply' CategoryTheory.Limits.Types.pi_lift_π_apply' /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`. -/ @[simp 1001] theorem pi_map_π_apply {β : Type v} [Small.{u} β] {f g : β → Type u} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := Limit.map_π_apply.{v, u} _ _ _ #align category_theory.limits.types.pi_map_π_apply CategoryTheory.Limits.Types.pi_map_π_apply /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`, with specialized universes. -/ theorem pi_map_π_apply' {β : Type v} {f g : β → Type v} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := by simp #align category_theory.limits.types.pi_map_π_apply' CategoryTheory.Limits.Types.pi_map_π_apply' /-- The category of types has `PUnit` as a terminal object. -/ def terminalLimitCone : Limits.LimitCone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cone := { pt := PUnit π := (Functor.uniqueFromEmpty _).hom } isLimit := { lift := fun _ _ => PUnit.unit fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext apply Subsingleton.elim } #align category_theory.limits.types.terminal_limit_cone CategoryTheory.Limits.Types.terminalLimitCone /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def terminalIso : ⊤_ Type u ≅ PUnit := limit.isoLimitCone terminalLimitCone.{u, 0} #align category_theory.limits.types.terminal_iso CategoryTheory.Limits.Types.terminalIso /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def isTerminalPunit : IsTerminal (PUnit : Type u) := terminalIsTerminal.ofIso terminalIso #align category_theory.limits.types.is_terminal_punit CategoryTheory.Limits.Types.isTerminalPunit -- porting note: the following three instances have been added to ease -- the automation in a definition in `AlgebraicTopology.SimplicialSet` noncomputable instance : Inhabited (⊤_ (Type u)) := ⟨@terminal.from (Type u) _ _ (ULift (Fin 1)) (ULift.up 0)⟩ instance : Subsingleton (⊤_ (Type u)) := ⟨fun a b => congr_fun (@Subsingleton.elim (_ ⟶ ⊤_ (Type u)) _ (fun _ => a) (fun _ => b)) (ULift.up (0 : Fin 1))⟩ noncomputable instance : Unique (⊤_ (Type u)) := Unique.mk' _ /-- A type is terminal if and only if it contains exactly one element. -/ noncomputable def isTerminalEquivUnique (X : Type u) : IsTerminal X ≃ Unique X := equivOfSubsingletonOfSubsingleton (fun h => ((Iso.toEquiv (terminalIsoIsTerminal h).symm).unique)) (fun _ => IsTerminal.ofIso terminalIsTerminal (Equiv.toIso (Equiv.equivOfUnique _ _))) /-- A type is terminal if and only if it is isomorphic to `PUnit`. -/ noncomputable def isTerminalEquivIsoPUnit (X : Type u) : IsTerminal X ≃ (X ≅ PUnit) := by calc IsTerminal X ≃ Unique X := isTerminalEquivUnique _ _ ≃ (X ≃ PUnit.{u + 1}) := uniqueEquivEquivUnique _ _ _ ≃ (X ≅ PUnit) := equivEquivIso /-- The category of types has `PEmpty` as an initial object. -/ def initialColimitCocone : Limits.ColimitCocone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cocone := { pt := PEmpty ι := (Functor.uniqueFromEmpty _).inv } isColimit := { desc := fun _ => by rintro ⟨⟩ fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext x; cases x } #align category_theory.limits.types.initial_colimit_cocone CategoryTheory.Limits.Types.initialColimitCocone /-- The initial object in `Type u` is `PEmpty`. -/ noncomputable def initialIso : ⊥_ Type u ≅ PEmpty := colimit.isoColimitCocone initialColimitCocone.{u, 0} #align category_theory.limits.types.initial_iso CategoryTheory.Limits.Types.initialIso /-- The initial object in `Type u` is `PEmpty`. -/ noncomputable def isInitialPunit : IsInitial (PEmpty : Type u) := initialIsInitial.ofIso initialIso #align category_theory.limits.types.is_initial_punit CategoryTheory.Limits.Types.isInitialPunit open CategoryTheory.Limits.WalkingPair -- We manually generate the other projection lemmas since the simp-normal form for the legs is -- otherwise not created correctly. /-- The product type `X × Y` forms a cone for the binary product of `X` and `Y`. -/ @[simps! pt] def binaryProductCone (X Y : Type u) : BinaryFan X Y := BinaryFan.mk _root_.Prod.fst _root_.Prod.snd #align category_theory.limits.types.binary_product_cone CategoryTheory.Limits.Types.binaryProductCone @[simp] theorem binaryProductCone_fst (X Y : Type u) : (binaryProductCone X Y).fst = _root_.Prod.fst := rfl #align category_theory.limits.types.binary_product_cone_fst CategoryTheory.Limits.Types.binaryProductCone_fst @[simp] theorem binaryProductCone_snd (X Y : Type u) : (binaryProductCone X Y).snd = _root_.Prod.snd := rfl #align category_theory.limits.types.binary_product_cone_snd CategoryTheory.Limits.Types.binaryProductCone_snd /-- The product type `X × Y` is a binary product for `X` and `Y`. -/ @[simps] def binaryProductLimit (X Y : Type u) : IsLimit (binaryProductCone X Y) where lift (s : BinaryFan X Y) x := (s.fst x, s.snd x) fac _ j := Discrete.recOn j fun j => WalkingPair.casesOn j rfl rfl uniq _ _ w := funext fun x => Prod.ext (congr_fun (w ⟨left⟩) x) (congr_fun (w ⟨right⟩) x) #align category_theory.limits.types.binary_product_limit CategoryTheory.Limits.Types.binaryProductLimit /-- The category of types has `X × Y`, the usual cartesian product, as the binary product of `X` and `Y`. -/ @[simps] def binaryProductLimitCone (X Y : Type u) : Limits.LimitCone (pair X Y) := ⟨_, binaryProductLimit X Y⟩ #align category_theory.limits.types.binary_product_limit_cone CategoryTheory.Limits.Types.binaryProductLimitCone /-- The categorical binary product in `Type u` is cartesian product. -/ noncomputable def binaryProductIso (X Y : Type u) : Limits.prod X Y ≅ X × Y := limit.isoLimitCone (binaryProductLimitCone X Y) #align category_theory.limits.types.binary_product_iso CategoryTheory.Limits.Types.binaryProductIso @[elementwise (attr := simp)] theorem binaryProductIso_hom_comp_fst (X Y : Type u) : (binaryProductIso X Y).hom ≫ _root_.Prod.fst = Limits.prod.fst := limit.isoLimitCone_hom_π (binaryProductLimitCone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_product_iso_hom_comp_fst CategoryTheory.Limits.Types.binaryProductIso_hom_comp_fst @[elementwise (attr := simp)] theorem binaryProductIso_hom_comp_snd (X Y : Type u) : (binaryProductIso X Y).hom ≫ _root_.Prod.snd = Limits.prod.snd := limit.isoLimitCone_hom_π (binaryProductLimitCone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_product_iso_hom_comp_snd CategoryTheory.Limits.Types.binaryProductIso_hom_comp_snd @[elementwise (attr := simp)] theorem binaryProductIso_inv_comp_fst (X Y : Type u) : (binaryProductIso X Y).inv ≫ Limits.prod.fst = _root_.Prod.fst := limit.isoLimitCone_inv_π (binaryProductLimitCone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_product_iso_inv_comp_fst CategoryTheory.Limits.Types.binaryProductIso_inv_comp_fst @[elementwise (attr := simp)] theorem binaryProductIso_inv_comp_snd (X Y : Type u) : (binaryProductIso X Y).inv ≫ Limits.prod.snd = _root_.Prod.snd := limit.isoLimitCone_inv_π (binaryProductLimitCone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_product_iso_inv_comp_snd CategoryTheory.Limits.Types.binaryProductIso_inv_comp_snd -- porting note: it was originally @[simps (config := { typeMd := reducible })] -- We add the option `type_md` to tell `@[simps]` to not treat homomorphisms `X ⟶ Y` in `Type*` as -- a function type /-- The functor which sends `X, Y` to the product type `X × Y`. -/ @[simps] def binaryProductFunctor : Type u ⥤ Type u ⥤ Type u where obj X := { obj := fun Y => X × Y map := fun { Y₁ Y₂} f => (binaryProductLimit X Y₂).lift (BinaryFan.mk _root_.Prod.fst (_root_.Prod.snd ≫ f)) } map {X₁ X₂} f := { app := fun Y => (binaryProductLimit X₂ Y).lift (BinaryFan.mk (_root_.Prod.fst ≫ f) _root_.Prod.snd) } #align category_theory.limits.types.binary_product_functor CategoryTheory.Limits.Types.binaryProductFunctor /-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _) := by refine' NatIso.ofComponents (fun X => _) (fun _ => _) · refine' NatIso.ofComponents (fun Y => _) (fun _ => _) · exact ((limit.isLimit _).conePointUniqueUpToIso (binaryProductLimit X Y)).symm · apply Limits.prod.hom_ext <;> simp <;> rfl · ext : 2 apply Limits.prod.hom_ext <;> simp <;> rfl #align category_theory.limits.types.binary_product_iso_prod CategoryTheory.Limits.Types.binaryProductIsoProd /-- The sum type `X ⊕ Y` forms a cocone for the binary coproduct of `X` and `Y`. -/ @[simps!] def binaryCoproductCocone (X Y : Type u) : Cocone (pair X Y) := BinaryCofan.mk Sum.inl Sum.inr #align category_theory.limits.types.binary_coproduct_cocone CategoryTheory.Limits.Types.binaryCoproductCocone /-- The sum type `X ⊕ Y` is a binary coproduct for `X` and `Y`. -/ @[simps] def binaryCoproductColimit (X Y : Type u) : IsColimit (binaryCoproductCocone X Y) where desc := fun s : BinaryCofan X Y => Sum.elim s.inl s.inr fac _ j := Discrete.recOn j fun j => WalkingPair.casesOn j rfl rfl uniq _ _ w := funext fun x => Sum.casesOn x (congr_fun (w ⟨left⟩)) (congr_fun (w ⟨right⟩)) #align category_theory.limits.types.binary_coproduct_colimit CategoryTheory.Limits.Types.binaryCoproductColimit /-- The category of types has `X ⊕ Y`, as the binary coproduct of `X` and `Y`. -/ def binaryCoproductColimitCocone (X Y : Type u) : Limits.ColimitCocone (pair X Y) := ⟨_, binaryCoproductColimit X Y⟩ #align category_theory.limits.types.binary_coproduct_colimit_cocone CategoryTheory.Limits.Types.binaryCoproductColimitCocone /-- The categorical binary coproduct in `Type u` is the sum `X ⊕ Y`. -/ noncomputable def binaryCoproductIso (X Y : Type u) : Limits.coprod X Y ≅ Sum X Y := colimit.isoColimitCocone (binaryCoproductColimitCocone X Y) #align category_theory.limits.types.binary_coproduct_iso CategoryTheory.Limits.Types.binaryCoproductIso --open CategoryTheory.Type @[elementwise (attr := simp)] theorem binaryCoproductIso_inl_comp_hom (X Y : Type u) : Limits.coprod.inl ≫ (binaryCoproductIso X Y).hom = Sum.inl := colimit.isoColimitCocone_ι_hom (binaryCoproductColimitCocone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_coproduct_iso_inl_comp_hom CategoryTheory.Limits.Types.binaryCoproductIso_inl_comp_hom @[elementwise (attr := simp)] theorem binaryCoproductIso_inr_comp_hom (X Y : Type u) : Limits.coprod.inr ≫ (binaryCoproductIso X Y).hom = Sum.inr := colimit.isoColimitCocone_ι_hom (binaryCoproductColimitCocone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_coproduct_iso_inr_comp_hom CategoryTheory.Limits.Types.binaryCoproductIso_inr_comp_hom @[elementwise (attr := simp)] theorem binaryCoproductIso_inl_comp_inv (X Y : Type u) : ↾(Sum.inl : X ⟶ Sum X Y) ≫ (binaryCoproductIso X Y).inv = Limits.coprod.inl := colimit.isoColimitCocone_ι_inv (binaryCoproductColimitCocone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_coproduct_iso_inl_comp_inv CategoryTheory.Limits.Types.binaryCoproductIso_inl_comp_inv @[elementwise (attr := simp)] theorem binaryCoproductIso_inr_comp_inv (X Y : Type u) : ↾(Sum.inr : Y ⟶ Sum X Y) ≫ (binaryCoproductIso X Y).inv = Limits.coprod.inr := colimit.isoColimitCocone_ι_inv (binaryCoproductColimitCocone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_coproduct_iso_inr_comp_inv CategoryTheory.Limits.Types.binaryCoproductIso_inr_comp_inv open Function (Injective) theorem binaryCofan_isColimit_iff {X Y : Type u} (c : BinaryCofan X Y) : Nonempty (IsColimit c) ↔ Injective c.inl ∧ Injective c.inr ∧ IsCompl (Set.range c.inl) (Set.range c.inr) := by classical constructor ·
rintro ⟨h⟩
theorem binaryCofan_isColimit_iff {X Y : Type u} (c : BinaryCofan X Y) : Nonempty (IsColimit c) ↔ Injective c.inl ∧ Injective c.inr ∧ IsCompl (Set.range c.inl) (Set.range c.inr) := by classical constructor ·
Mathlib.CategoryTheory.Limits.Shapes.Types.302_0.ctQAUYXLRXnvMGw
theorem binaryCofan_isColimit_iff {X Y : Type u} (c : BinaryCofan X Y) : Nonempty (IsColimit c) ↔ Injective c.inl ∧ Injective c.inr ∧ IsCompl (Set.range c.inl) (Set.range c.inr)
Mathlib_CategoryTheory_Limits_Shapes_Types
case mp.intro X Y : Type u c : BinaryCofan X Y h : IsColimit c ⊢ Injective (BinaryCofan.inl c) ∧ Injective (BinaryCofan.inr c) ∧ IsCompl (Set.range (BinaryCofan.inl c)) (Set.range (BinaryCofan.inr c))
/- Copyright (c) 2020 Scott Morrison. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Scott Morrison -/ import Mathlib.CategoryTheory.Limits.Types import Mathlib.CategoryTheory.Limits.Shapes.Products import Mathlib.CategoryTheory.Limits.Shapes.BinaryProducts import Mathlib.CategoryTheory.Limits.Shapes.Terminal import Mathlib.CategoryTheory.ConcreteCategory.Basic import Mathlib.Tactic.CategoryTheory.Elementwise #align_import category_theory.limits.shapes.types from "leanprover-community/mathlib"@"5dc6092d09e5e489106865241986f7f2ad28d4c8" /-! # Special shapes for limits in `Type`. The general shape (co)limits defined in `CategoryTheory.Limits.Types` are intended for use through the limits API, and the actual implementation should mostly be considered "sealed". In this file, we provide definitions of the "standard" special shapes of limits in `Type`, giving the expected definitional implementation: * the terminal object is `PUnit` * the binary product of `X` and `Y` is `X × Y` * the product of a family `f : J → Type` is `Π j, f j` * the coproduct of a family `f : J → Type` is `Σ j, f j` * the binary coproduct of `X` and `Y` is the sum type `X ⊕ Y` * the equalizer of a pair of maps `(g, h)` is the subtype `{x : Y // g x = h x}` * the coequalizer of a pair of maps `(f, g)` is the quotient of `Y` by `∀ x : Y, f x ~ g x` * the pullback of `f : X ⟶ Z` and `g : Y ⟶ Z` is the subtype `{ p : X × Y // f p.1 = g p.2 }` of the product We first construct terms of `IsLimit` and `LimitCone`, and then provide isomorphisms with the types generated by the `HasLimit` API. As an example, when setting up the monoidal category structure on `Type` we use the `Types.terminalLimitCone` and `Types.binaryProductLimitCone` definitions. -/ universe v u open CategoryTheory Limits namespace CategoryTheory.Limits.Types example : HasProducts.{v} (Type v) := inferInstance example [UnivLE.{v, u}] : HasProducts.{v} (Type u) := inferInstance -- This shortcut instance is required in `Mathlib.CategoryTheory.Closed.Types`, -- although I don't understand why, and wish it wasn't. instance : HasProducts.{v} (Type v) := inferInstance /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`. -/ @[simp 1001] theorem pi_lift_π_apply {β : Type v} [Small.{u} β] (f : β → Type u) {P : Type u} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := congr_fun (limit.lift_π (Fan.mk P s) ⟨b⟩) x #align category_theory.limits.types.pi_lift_π_apply CategoryTheory.Limits.Types.pi_lift_π_apply /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`, with specialized universes. -/ theorem pi_lift_π_apply' {β : Type v} (f : β → Type v) {P : Type v} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := by simp #align category_theory.limits.types.pi_lift_π_apply' CategoryTheory.Limits.Types.pi_lift_π_apply' /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`. -/ @[simp 1001] theorem pi_map_π_apply {β : Type v} [Small.{u} β] {f g : β → Type u} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := Limit.map_π_apply.{v, u} _ _ _ #align category_theory.limits.types.pi_map_π_apply CategoryTheory.Limits.Types.pi_map_π_apply /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`, with specialized universes. -/ theorem pi_map_π_apply' {β : Type v} {f g : β → Type v} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := by simp #align category_theory.limits.types.pi_map_π_apply' CategoryTheory.Limits.Types.pi_map_π_apply' /-- The category of types has `PUnit` as a terminal object. -/ def terminalLimitCone : Limits.LimitCone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cone := { pt := PUnit π := (Functor.uniqueFromEmpty _).hom } isLimit := { lift := fun _ _ => PUnit.unit fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext apply Subsingleton.elim } #align category_theory.limits.types.terminal_limit_cone CategoryTheory.Limits.Types.terminalLimitCone /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def terminalIso : ⊤_ Type u ≅ PUnit := limit.isoLimitCone terminalLimitCone.{u, 0} #align category_theory.limits.types.terminal_iso CategoryTheory.Limits.Types.terminalIso /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def isTerminalPunit : IsTerminal (PUnit : Type u) := terminalIsTerminal.ofIso terminalIso #align category_theory.limits.types.is_terminal_punit CategoryTheory.Limits.Types.isTerminalPunit -- porting note: the following three instances have been added to ease -- the automation in a definition in `AlgebraicTopology.SimplicialSet` noncomputable instance : Inhabited (⊤_ (Type u)) := ⟨@terminal.from (Type u) _ _ (ULift (Fin 1)) (ULift.up 0)⟩ instance : Subsingleton (⊤_ (Type u)) := ⟨fun a b => congr_fun (@Subsingleton.elim (_ ⟶ ⊤_ (Type u)) _ (fun _ => a) (fun _ => b)) (ULift.up (0 : Fin 1))⟩ noncomputable instance : Unique (⊤_ (Type u)) := Unique.mk' _ /-- A type is terminal if and only if it contains exactly one element. -/ noncomputable def isTerminalEquivUnique (X : Type u) : IsTerminal X ≃ Unique X := equivOfSubsingletonOfSubsingleton (fun h => ((Iso.toEquiv (terminalIsoIsTerminal h).symm).unique)) (fun _ => IsTerminal.ofIso terminalIsTerminal (Equiv.toIso (Equiv.equivOfUnique _ _))) /-- A type is terminal if and only if it is isomorphic to `PUnit`. -/ noncomputable def isTerminalEquivIsoPUnit (X : Type u) : IsTerminal X ≃ (X ≅ PUnit) := by calc IsTerminal X ≃ Unique X := isTerminalEquivUnique _ _ ≃ (X ≃ PUnit.{u + 1}) := uniqueEquivEquivUnique _ _ _ ≃ (X ≅ PUnit) := equivEquivIso /-- The category of types has `PEmpty` as an initial object. -/ def initialColimitCocone : Limits.ColimitCocone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cocone := { pt := PEmpty ι := (Functor.uniqueFromEmpty _).inv } isColimit := { desc := fun _ => by rintro ⟨⟩ fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext x; cases x } #align category_theory.limits.types.initial_colimit_cocone CategoryTheory.Limits.Types.initialColimitCocone /-- The initial object in `Type u` is `PEmpty`. -/ noncomputable def initialIso : ⊥_ Type u ≅ PEmpty := colimit.isoColimitCocone initialColimitCocone.{u, 0} #align category_theory.limits.types.initial_iso CategoryTheory.Limits.Types.initialIso /-- The initial object in `Type u` is `PEmpty`. -/ noncomputable def isInitialPunit : IsInitial (PEmpty : Type u) := initialIsInitial.ofIso initialIso #align category_theory.limits.types.is_initial_punit CategoryTheory.Limits.Types.isInitialPunit open CategoryTheory.Limits.WalkingPair -- We manually generate the other projection lemmas since the simp-normal form for the legs is -- otherwise not created correctly. /-- The product type `X × Y` forms a cone for the binary product of `X` and `Y`. -/ @[simps! pt] def binaryProductCone (X Y : Type u) : BinaryFan X Y := BinaryFan.mk _root_.Prod.fst _root_.Prod.snd #align category_theory.limits.types.binary_product_cone CategoryTheory.Limits.Types.binaryProductCone @[simp] theorem binaryProductCone_fst (X Y : Type u) : (binaryProductCone X Y).fst = _root_.Prod.fst := rfl #align category_theory.limits.types.binary_product_cone_fst CategoryTheory.Limits.Types.binaryProductCone_fst @[simp] theorem binaryProductCone_snd (X Y : Type u) : (binaryProductCone X Y).snd = _root_.Prod.snd := rfl #align category_theory.limits.types.binary_product_cone_snd CategoryTheory.Limits.Types.binaryProductCone_snd /-- The product type `X × Y` is a binary product for `X` and `Y`. -/ @[simps] def binaryProductLimit (X Y : Type u) : IsLimit (binaryProductCone X Y) where lift (s : BinaryFan X Y) x := (s.fst x, s.snd x) fac _ j := Discrete.recOn j fun j => WalkingPair.casesOn j rfl rfl uniq _ _ w := funext fun x => Prod.ext (congr_fun (w ⟨left⟩) x) (congr_fun (w ⟨right⟩) x) #align category_theory.limits.types.binary_product_limit CategoryTheory.Limits.Types.binaryProductLimit /-- The category of types has `X × Y`, the usual cartesian product, as the binary product of `X` and `Y`. -/ @[simps] def binaryProductLimitCone (X Y : Type u) : Limits.LimitCone (pair X Y) := ⟨_, binaryProductLimit X Y⟩ #align category_theory.limits.types.binary_product_limit_cone CategoryTheory.Limits.Types.binaryProductLimitCone /-- The categorical binary product in `Type u` is cartesian product. -/ noncomputable def binaryProductIso (X Y : Type u) : Limits.prod X Y ≅ X × Y := limit.isoLimitCone (binaryProductLimitCone X Y) #align category_theory.limits.types.binary_product_iso CategoryTheory.Limits.Types.binaryProductIso @[elementwise (attr := simp)] theorem binaryProductIso_hom_comp_fst (X Y : Type u) : (binaryProductIso X Y).hom ≫ _root_.Prod.fst = Limits.prod.fst := limit.isoLimitCone_hom_π (binaryProductLimitCone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_product_iso_hom_comp_fst CategoryTheory.Limits.Types.binaryProductIso_hom_comp_fst @[elementwise (attr := simp)] theorem binaryProductIso_hom_comp_snd (X Y : Type u) : (binaryProductIso X Y).hom ≫ _root_.Prod.snd = Limits.prod.snd := limit.isoLimitCone_hom_π (binaryProductLimitCone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_product_iso_hom_comp_snd CategoryTheory.Limits.Types.binaryProductIso_hom_comp_snd @[elementwise (attr := simp)] theorem binaryProductIso_inv_comp_fst (X Y : Type u) : (binaryProductIso X Y).inv ≫ Limits.prod.fst = _root_.Prod.fst := limit.isoLimitCone_inv_π (binaryProductLimitCone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_product_iso_inv_comp_fst CategoryTheory.Limits.Types.binaryProductIso_inv_comp_fst @[elementwise (attr := simp)] theorem binaryProductIso_inv_comp_snd (X Y : Type u) : (binaryProductIso X Y).inv ≫ Limits.prod.snd = _root_.Prod.snd := limit.isoLimitCone_inv_π (binaryProductLimitCone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_product_iso_inv_comp_snd CategoryTheory.Limits.Types.binaryProductIso_inv_comp_snd -- porting note: it was originally @[simps (config := { typeMd := reducible })] -- We add the option `type_md` to tell `@[simps]` to not treat homomorphisms `X ⟶ Y` in `Type*` as -- a function type /-- The functor which sends `X, Y` to the product type `X × Y`. -/ @[simps] def binaryProductFunctor : Type u ⥤ Type u ⥤ Type u where obj X := { obj := fun Y => X × Y map := fun { Y₁ Y₂} f => (binaryProductLimit X Y₂).lift (BinaryFan.mk _root_.Prod.fst (_root_.Prod.snd ≫ f)) } map {X₁ X₂} f := { app := fun Y => (binaryProductLimit X₂ Y).lift (BinaryFan.mk (_root_.Prod.fst ≫ f) _root_.Prod.snd) } #align category_theory.limits.types.binary_product_functor CategoryTheory.Limits.Types.binaryProductFunctor /-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _) := by refine' NatIso.ofComponents (fun X => _) (fun _ => _) · refine' NatIso.ofComponents (fun Y => _) (fun _ => _) · exact ((limit.isLimit _).conePointUniqueUpToIso (binaryProductLimit X Y)).symm · apply Limits.prod.hom_ext <;> simp <;> rfl · ext : 2 apply Limits.prod.hom_ext <;> simp <;> rfl #align category_theory.limits.types.binary_product_iso_prod CategoryTheory.Limits.Types.binaryProductIsoProd /-- The sum type `X ⊕ Y` forms a cocone for the binary coproduct of `X` and `Y`. -/ @[simps!] def binaryCoproductCocone (X Y : Type u) : Cocone (pair X Y) := BinaryCofan.mk Sum.inl Sum.inr #align category_theory.limits.types.binary_coproduct_cocone CategoryTheory.Limits.Types.binaryCoproductCocone /-- The sum type `X ⊕ Y` is a binary coproduct for `X` and `Y`. -/ @[simps] def binaryCoproductColimit (X Y : Type u) : IsColimit (binaryCoproductCocone X Y) where desc := fun s : BinaryCofan X Y => Sum.elim s.inl s.inr fac _ j := Discrete.recOn j fun j => WalkingPair.casesOn j rfl rfl uniq _ _ w := funext fun x => Sum.casesOn x (congr_fun (w ⟨left⟩)) (congr_fun (w ⟨right⟩)) #align category_theory.limits.types.binary_coproduct_colimit CategoryTheory.Limits.Types.binaryCoproductColimit /-- The category of types has `X ⊕ Y`, as the binary coproduct of `X` and `Y`. -/ def binaryCoproductColimitCocone (X Y : Type u) : Limits.ColimitCocone (pair X Y) := ⟨_, binaryCoproductColimit X Y⟩ #align category_theory.limits.types.binary_coproduct_colimit_cocone CategoryTheory.Limits.Types.binaryCoproductColimitCocone /-- The categorical binary coproduct in `Type u` is the sum `X ⊕ Y`. -/ noncomputable def binaryCoproductIso (X Y : Type u) : Limits.coprod X Y ≅ Sum X Y := colimit.isoColimitCocone (binaryCoproductColimitCocone X Y) #align category_theory.limits.types.binary_coproduct_iso CategoryTheory.Limits.Types.binaryCoproductIso --open CategoryTheory.Type @[elementwise (attr := simp)] theorem binaryCoproductIso_inl_comp_hom (X Y : Type u) : Limits.coprod.inl ≫ (binaryCoproductIso X Y).hom = Sum.inl := colimit.isoColimitCocone_ι_hom (binaryCoproductColimitCocone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_coproduct_iso_inl_comp_hom CategoryTheory.Limits.Types.binaryCoproductIso_inl_comp_hom @[elementwise (attr := simp)] theorem binaryCoproductIso_inr_comp_hom (X Y : Type u) : Limits.coprod.inr ≫ (binaryCoproductIso X Y).hom = Sum.inr := colimit.isoColimitCocone_ι_hom (binaryCoproductColimitCocone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_coproduct_iso_inr_comp_hom CategoryTheory.Limits.Types.binaryCoproductIso_inr_comp_hom @[elementwise (attr := simp)] theorem binaryCoproductIso_inl_comp_inv (X Y : Type u) : ↾(Sum.inl : X ⟶ Sum X Y) ≫ (binaryCoproductIso X Y).inv = Limits.coprod.inl := colimit.isoColimitCocone_ι_inv (binaryCoproductColimitCocone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_coproduct_iso_inl_comp_inv CategoryTheory.Limits.Types.binaryCoproductIso_inl_comp_inv @[elementwise (attr := simp)] theorem binaryCoproductIso_inr_comp_inv (X Y : Type u) : ↾(Sum.inr : Y ⟶ Sum X Y) ≫ (binaryCoproductIso X Y).inv = Limits.coprod.inr := colimit.isoColimitCocone_ι_inv (binaryCoproductColimitCocone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_coproduct_iso_inr_comp_inv CategoryTheory.Limits.Types.binaryCoproductIso_inr_comp_inv open Function (Injective) theorem binaryCofan_isColimit_iff {X Y : Type u} (c : BinaryCofan X Y) : Nonempty (IsColimit c) ↔ Injective c.inl ∧ Injective c.inr ∧ IsCompl (Set.range c.inl) (Set.range c.inr) := by classical constructor · rintro ⟨h⟩
rw [← show _ = c.inl from h.comp_coconePointUniqueUpToIso_inv (binaryCoproductColimit X Y) ⟨WalkingPair.left⟩, ← show _ = c.inr from h.comp_coconePointUniqueUpToIso_inv (binaryCoproductColimit X Y) ⟨WalkingPair.right⟩]
theorem binaryCofan_isColimit_iff {X Y : Type u} (c : BinaryCofan X Y) : Nonempty (IsColimit c) ↔ Injective c.inl ∧ Injective c.inr ∧ IsCompl (Set.range c.inl) (Set.range c.inr) := by classical constructor · rintro ⟨h⟩
Mathlib.CategoryTheory.Limits.Shapes.Types.302_0.ctQAUYXLRXnvMGw
theorem binaryCofan_isColimit_iff {X Y : Type u} (c : BinaryCofan X Y) : Nonempty (IsColimit c) ↔ Injective c.inl ∧ Injective c.inr ∧ IsCompl (Set.range c.inl) (Set.range c.inr)
Mathlib_CategoryTheory_Limits_Shapes_Types
case mp.intro X Y : Type u c : BinaryCofan X Y h : IsColimit c ⊢ Injective ((binaryCoproductCocone X Y).ι.app { as := left } ≫ (IsColimit.coconePointUniqueUpToIso h (binaryCoproductColimit X Y)).inv) ∧ Injective ((binaryCoproductCocone X Y).ι.app { as := right } ≫ (IsColimit.coconePointUniqueUpToIso h (binaryCoproductColimit X Y)).inv) ∧ IsCompl (Set.range ((binaryCoproductCocone X Y).ι.app { as := left } ≫ (IsColimit.coconePointUniqueUpToIso h (binaryCoproductColimit X Y)).inv)) (Set.range ((binaryCoproductCocone X Y).ι.app { as := right } ≫ (IsColimit.coconePointUniqueUpToIso h (binaryCoproductColimit X Y)).inv))
/- Copyright (c) 2020 Scott Morrison. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Scott Morrison -/ import Mathlib.CategoryTheory.Limits.Types import Mathlib.CategoryTheory.Limits.Shapes.Products import Mathlib.CategoryTheory.Limits.Shapes.BinaryProducts import Mathlib.CategoryTheory.Limits.Shapes.Terminal import Mathlib.CategoryTheory.ConcreteCategory.Basic import Mathlib.Tactic.CategoryTheory.Elementwise #align_import category_theory.limits.shapes.types from "leanprover-community/mathlib"@"5dc6092d09e5e489106865241986f7f2ad28d4c8" /-! # Special shapes for limits in `Type`. The general shape (co)limits defined in `CategoryTheory.Limits.Types` are intended for use through the limits API, and the actual implementation should mostly be considered "sealed". In this file, we provide definitions of the "standard" special shapes of limits in `Type`, giving the expected definitional implementation: * the terminal object is `PUnit` * the binary product of `X` and `Y` is `X × Y` * the product of a family `f : J → Type` is `Π j, f j` * the coproduct of a family `f : J → Type` is `Σ j, f j` * the binary coproduct of `X` and `Y` is the sum type `X ⊕ Y` * the equalizer of a pair of maps `(g, h)` is the subtype `{x : Y // g x = h x}` * the coequalizer of a pair of maps `(f, g)` is the quotient of `Y` by `∀ x : Y, f x ~ g x` * the pullback of `f : X ⟶ Z` and `g : Y ⟶ Z` is the subtype `{ p : X × Y // f p.1 = g p.2 }` of the product We first construct terms of `IsLimit` and `LimitCone`, and then provide isomorphisms with the types generated by the `HasLimit` API. As an example, when setting up the monoidal category structure on `Type` we use the `Types.terminalLimitCone` and `Types.binaryProductLimitCone` definitions. -/ universe v u open CategoryTheory Limits namespace CategoryTheory.Limits.Types example : HasProducts.{v} (Type v) := inferInstance example [UnivLE.{v, u}] : HasProducts.{v} (Type u) := inferInstance -- This shortcut instance is required in `Mathlib.CategoryTheory.Closed.Types`, -- although I don't understand why, and wish it wasn't. instance : HasProducts.{v} (Type v) := inferInstance /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`. -/ @[simp 1001] theorem pi_lift_π_apply {β : Type v} [Small.{u} β] (f : β → Type u) {P : Type u} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := congr_fun (limit.lift_π (Fan.mk P s) ⟨b⟩) x #align category_theory.limits.types.pi_lift_π_apply CategoryTheory.Limits.Types.pi_lift_π_apply /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`, with specialized universes. -/ theorem pi_lift_π_apply' {β : Type v} (f : β → Type v) {P : Type v} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := by simp #align category_theory.limits.types.pi_lift_π_apply' CategoryTheory.Limits.Types.pi_lift_π_apply' /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`. -/ @[simp 1001] theorem pi_map_π_apply {β : Type v} [Small.{u} β] {f g : β → Type u} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := Limit.map_π_apply.{v, u} _ _ _ #align category_theory.limits.types.pi_map_π_apply CategoryTheory.Limits.Types.pi_map_π_apply /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`, with specialized universes. -/ theorem pi_map_π_apply' {β : Type v} {f g : β → Type v} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := by simp #align category_theory.limits.types.pi_map_π_apply' CategoryTheory.Limits.Types.pi_map_π_apply' /-- The category of types has `PUnit` as a terminal object. -/ def terminalLimitCone : Limits.LimitCone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cone := { pt := PUnit π := (Functor.uniqueFromEmpty _).hom } isLimit := { lift := fun _ _ => PUnit.unit fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext apply Subsingleton.elim } #align category_theory.limits.types.terminal_limit_cone CategoryTheory.Limits.Types.terminalLimitCone /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def terminalIso : ⊤_ Type u ≅ PUnit := limit.isoLimitCone terminalLimitCone.{u, 0} #align category_theory.limits.types.terminal_iso CategoryTheory.Limits.Types.terminalIso /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def isTerminalPunit : IsTerminal (PUnit : Type u) := terminalIsTerminal.ofIso terminalIso #align category_theory.limits.types.is_terminal_punit CategoryTheory.Limits.Types.isTerminalPunit -- porting note: the following three instances have been added to ease -- the automation in a definition in `AlgebraicTopology.SimplicialSet` noncomputable instance : Inhabited (⊤_ (Type u)) := ⟨@terminal.from (Type u) _ _ (ULift (Fin 1)) (ULift.up 0)⟩ instance : Subsingleton (⊤_ (Type u)) := ⟨fun a b => congr_fun (@Subsingleton.elim (_ ⟶ ⊤_ (Type u)) _ (fun _ => a) (fun _ => b)) (ULift.up (0 : Fin 1))⟩ noncomputable instance : Unique (⊤_ (Type u)) := Unique.mk' _ /-- A type is terminal if and only if it contains exactly one element. -/ noncomputable def isTerminalEquivUnique (X : Type u) : IsTerminal X ≃ Unique X := equivOfSubsingletonOfSubsingleton (fun h => ((Iso.toEquiv (terminalIsoIsTerminal h).symm).unique)) (fun _ => IsTerminal.ofIso terminalIsTerminal (Equiv.toIso (Equiv.equivOfUnique _ _))) /-- A type is terminal if and only if it is isomorphic to `PUnit`. -/ noncomputable def isTerminalEquivIsoPUnit (X : Type u) : IsTerminal X ≃ (X ≅ PUnit) := by calc IsTerminal X ≃ Unique X := isTerminalEquivUnique _ _ ≃ (X ≃ PUnit.{u + 1}) := uniqueEquivEquivUnique _ _ _ ≃ (X ≅ PUnit) := equivEquivIso /-- The category of types has `PEmpty` as an initial object. -/ def initialColimitCocone : Limits.ColimitCocone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cocone := { pt := PEmpty ι := (Functor.uniqueFromEmpty _).inv } isColimit := { desc := fun _ => by rintro ⟨⟩ fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext x; cases x } #align category_theory.limits.types.initial_colimit_cocone CategoryTheory.Limits.Types.initialColimitCocone /-- The initial object in `Type u` is `PEmpty`. -/ noncomputable def initialIso : ⊥_ Type u ≅ PEmpty := colimit.isoColimitCocone initialColimitCocone.{u, 0} #align category_theory.limits.types.initial_iso CategoryTheory.Limits.Types.initialIso /-- The initial object in `Type u` is `PEmpty`. -/ noncomputable def isInitialPunit : IsInitial (PEmpty : Type u) := initialIsInitial.ofIso initialIso #align category_theory.limits.types.is_initial_punit CategoryTheory.Limits.Types.isInitialPunit open CategoryTheory.Limits.WalkingPair -- We manually generate the other projection lemmas since the simp-normal form for the legs is -- otherwise not created correctly. /-- The product type `X × Y` forms a cone for the binary product of `X` and `Y`. -/ @[simps! pt] def binaryProductCone (X Y : Type u) : BinaryFan X Y := BinaryFan.mk _root_.Prod.fst _root_.Prod.snd #align category_theory.limits.types.binary_product_cone CategoryTheory.Limits.Types.binaryProductCone @[simp] theorem binaryProductCone_fst (X Y : Type u) : (binaryProductCone X Y).fst = _root_.Prod.fst := rfl #align category_theory.limits.types.binary_product_cone_fst CategoryTheory.Limits.Types.binaryProductCone_fst @[simp] theorem binaryProductCone_snd (X Y : Type u) : (binaryProductCone X Y).snd = _root_.Prod.snd := rfl #align category_theory.limits.types.binary_product_cone_snd CategoryTheory.Limits.Types.binaryProductCone_snd /-- The product type `X × Y` is a binary product for `X` and `Y`. -/ @[simps] def binaryProductLimit (X Y : Type u) : IsLimit (binaryProductCone X Y) where lift (s : BinaryFan X Y) x := (s.fst x, s.snd x) fac _ j := Discrete.recOn j fun j => WalkingPair.casesOn j rfl rfl uniq _ _ w := funext fun x => Prod.ext (congr_fun (w ⟨left⟩) x) (congr_fun (w ⟨right⟩) x) #align category_theory.limits.types.binary_product_limit CategoryTheory.Limits.Types.binaryProductLimit /-- The category of types has `X × Y`, the usual cartesian product, as the binary product of `X` and `Y`. -/ @[simps] def binaryProductLimitCone (X Y : Type u) : Limits.LimitCone (pair X Y) := ⟨_, binaryProductLimit X Y⟩ #align category_theory.limits.types.binary_product_limit_cone CategoryTheory.Limits.Types.binaryProductLimitCone /-- The categorical binary product in `Type u` is cartesian product. -/ noncomputable def binaryProductIso (X Y : Type u) : Limits.prod X Y ≅ X × Y := limit.isoLimitCone (binaryProductLimitCone X Y) #align category_theory.limits.types.binary_product_iso CategoryTheory.Limits.Types.binaryProductIso @[elementwise (attr := simp)] theorem binaryProductIso_hom_comp_fst (X Y : Type u) : (binaryProductIso X Y).hom ≫ _root_.Prod.fst = Limits.prod.fst := limit.isoLimitCone_hom_π (binaryProductLimitCone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_product_iso_hom_comp_fst CategoryTheory.Limits.Types.binaryProductIso_hom_comp_fst @[elementwise (attr := simp)] theorem binaryProductIso_hom_comp_snd (X Y : Type u) : (binaryProductIso X Y).hom ≫ _root_.Prod.snd = Limits.prod.snd := limit.isoLimitCone_hom_π (binaryProductLimitCone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_product_iso_hom_comp_snd CategoryTheory.Limits.Types.binaryProductIso_hom_comp_snd @[elementwise (attr := simp)] theorem binaryProductIso_inv_comp_fst (X Y : Type u) : (binaryProductIso X Y).inv ≫ Limits.prod.fst = _root_.Prod.fst := limit.isoLimitCone_inv_π (binaryProductLimitCone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_product_iso_inv_comp_fst CategoryTheory.Limits.Types.binaryProductIso_inv_comp_fst @[elementwise (attr := simp)] theorem binaryProductIso_inv_comp_snd (X Y : Type u) : (binaryProductIso X Y).inv ≫ Limits.prod.snd = _root_.Prod.snd := limit.isoLimitCone_inv_π (binaryProductLimitCone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_product_iso_inv_comp_snd CategoryTheory.Limits.Types.binaryProductIso_inv_comp_snd -- porting note: it was originally @[simps (config := { typeMd := reducible })] -- We add the option `type_md` to tell `@[simps]` to not treat homomorphisms `X ⟶ Y` in `Type*` as -- a function type /-- The functor which sends `X, Y` to the product type `X × Y`. -/ @[simps] def binaryProductFunctor : Type u ⥤ Type u ⥤ Type u where obj X := { obj := fun Y => X × Y map := fun { Y₁ Y₂} f => (binaryProductLimit X Y₂).lift (BinaryFan.mk _root_.Prod.fst (_root_.Prod.snd ≫ f)) } map {X₁ X₂} f := { app := fun Y => (binaryProductLimit X₂ Y).lift (BinaryFan.mk (_root_.Prod.fst ≫ f) _root_.Prod.snd) } #align category_theory.limits.types.binary_product_functor CategoryTheory.Limits.Types.binaryProductFunctor /-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _) := by refine' NatIso.ofComponents (fun X => _) (fun _ => _) · refine' NatIso.ofComponents (fun Y => _) (fun _ => _) · exact ((limit.isLimit _).conePointUniqueUpToIso (binaryProductLimit X Y)).symm · apply Limits.prod.hom_ext <;> simp <;> rfl · ext : 2 apply Limits.prod.hom_ext <;> simp <;> rfl #align category_theory.limits.types.binary_product_iso_prod CategoryTheory.Limits.Types.binaryProductIsoProd /-- The sum type `X ⊕ Y` forms a cocone for the binary coproduct of `X` and `Y`. -/ @[simps!] def binaryCoproductCocone (X Y : Type u) : Cocone (pair X Y) := BinaryCofan.mk Sum.inl Sum.inr #align category_theory.limits.types.binary_coproduct_cocone CategoryTheory.Limits.Types.binaryCoproductCocone /-- The sum type `X ⊕ Y` is a binary coproduct for `X` and `Y`. -/ @[simps] def binaryCoproductColimit (X Y : Type u) : IsColimit (binaryCoproductCocone X Y) where desc := fun s : BinaryCofan X Y => Sum.elim s.inl s.inr fac _ j := Discrete.recOn j fun j => WalkingPair.casesOn j rfl rfl uniq _ _ w := funext fun x => Sum.casesOn x (congr_fun (w ⟨left⟩)) (congr_fun (w ⟨right⟩)) #align category_theory.limits.types.binary_coproduct_colimit CategoryTheory.Limits.Types.binaryCoproductColimit /-- The category of types has `X ⊕ Y`, as the binary coproduct of `X` and `Y`. -/ def binaryCoproductColimitCocone (X Y : Type u) : Limits.ColimitCocone (pair X Y) := ⟨_, binaryCoproductColimit X Y⟩ #align category_theory.limits.types.binary_coproduct_colimit_cocone CategoryTheory.Limits.Types.binaryCoproductColimitCocone /-- The categorical binary coproduct in `Type u` is the sum `X ⊕ Y`. -/ noncomputable def binaryCoproductIso (X Y : Type u) : Limits.coprod X Y ≅ Sum X Y := colimit.isoColimitCocone (binaryCoproductColimitCocone X Y) #align category_theory.limits.types.binary_coproduct_iso CategoryTheory.Limits.Types.binaryCoproductIso --open CategoryTheory.Type @[elementwise (attr := simp)] theorem binaryCoproductIso_inl_comp_hom (X Y : Type u) : Limits.coprod.inl ≫ (binaryCoproductIso X Y).hom = Sum.inl := colimit.isoColimitCocone_ι_hom (binaryCoproductColimitCocone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_coproduct_iso_inl_comp_hom CategoryTheory.Limits.Types.binaryCoproductIso_inl_comp_hom @[elementwise (attr := simp)] theorem binaryCoproductIso_inr_comp_hom (X Y : Type u) : Limits.coprod.inr ≫ (binaryCoproductIso X Y).hom = Sum.inr := colimit.isoColimitCocone_ι_hom (binaryCoproductColimitCocone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_coproduct_iso_inr_comp_hom CategoryTheory.Limits.Types.binaryCoproductIso_inr_comp_hom @[elementwise (attr := simp)] theorem binaryCoproductIso_inl_comp_inv (X Y : Type u) : ↾(Sum.inl : X ⟶ Sum X Y) ≫ (binaryCoproductIso X Y).inv = Limits.coprod.inl := colimit.isoColimitCocone_ι_inv (binaryCoproductColimitCocone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_coproduct_iso_inl_comp_inv CategoryTheory.Limits.Types.binaryCoproductIso_inl_comp_inv @[elementwise (attr := simp)] theorem binaryCoproductIso_inr_comp_inv (X Y : Type u) : ↾(Sum.inr : Y ⟶ Sum X Y) ≫ (binaryCoproductIso X Y).inv = Limits.coprod.inr := colimit.isoColimitCocone_ι_inv (binaryCoproductColimitCocone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_coproduct_iso_inr_comp_inv CategoryTheory.Limits.Types.binaryCoproductIso_inr_comp_inv open Function (Injective) theorem binaryCofan_isColimit_iff {X Y : Type u} (c : BinaryCofan X Y) : Nonempty (IsColimit c) ↔ Injective c.inl ∧ Injective c.inr ∧ IsCompl (Set.range c.inl) (Set.range c.inr) := by classical constructor · rintro ⟨h⟩ rw [← show _ = c.inl from h.comp_coconePointUniqueUpToIso_inv (binaryCoproductColimit X Y) ⟨WalkingPair.left⟩, ← show _ = c.inr from h.comp_coconePointUniqueUpToIso_inv (binaryCoproductColimit X Y) ⟨WalkingPair.right⟩]
dsimp [binaryCoproductCocone]
theorem binaryCofan_isColimit_iff {X Y : Type u} (c : BinaryCofan X Y) : Nonempty (IsColimit c) ↔ Injective c.inl ∧ Injective c.inr ∧ IsCompl (Set.range c.inl) (Set.range c.inr) := by classical constructor · rintro ⟨h⟩ rw [← show _ = c.inl from h.comp_coconePointUniqueUpToIso_inv (binaryCoproductColimit X Y) ⟨WalkingPair.left⟩, ← show _ = c.inr from h.comp_coconePointUniqueUpToIso_inv (binaryCoproductColimit X Y) ⟨WalkingPair.right⟩]
Mathlib.CategoryTheory.Limits.Shapes.Types.302_0.ctQAUYXLRXnvMGw
theorem binaryCofan_isColimit_iff {X Y : Type u} (c : BinaryCofan X Y) : Nonempty (IsColimit c) ↔ Injective c.inl ∧ Injective c.inr ∧ IsCompl (Set.range c.inl) (Set.range c.inr)
Mathlib_CategoryTheory_Limits_Shapes_Types
case mp.intro X Y : Type u c : BinaryCofan X Y h : IsColimit c ⊢ Injective (Sum.inl ≫ (IsColimit.coconePointUniqueUpToIso h (binaryCoproductColimit X Y)).inv) ∧ Injective (Sum.inr ≫ (IsColimit.coconePointUniqueUpToIso h (binaryCoproductColimit X Y)).inv) ∧ IsCompl (Set.range (Sum.inl ≫ (IsColimit.coconePointUniqueUpToIso h (binaryCoproductColimit X Y)).inv)) (Set.range (Sum.inr ≫ (IsColimit.coconePointUniqueUpToIso h (binaryCoproductColimit X Y)).inv))
/- Copyright (c) 2020 Scott Morrison. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Scott Morrison -/ import Mathlib.CategoryTheory.Limits.Types import Mathlib.CategoryTheory.Limits.Shapes.Products import Mathlib.CategoryTheory.Limits.Shapes.BinaryProducts import Mathlib.CategoryTheory.Limits.Shapes.Terminal import Mathlib.CategoryTheory.ConcreteCategory.Basic import Mathlib.Tactic.CategoryTheory.Elementwise #align_import category_theory.limits.shapes.types from "leanprover-community/mathlib"@"5dc6092d09e5e489106865241986f7f2ad28d4c8" /-! # Special shapes for limits in `Type`. The general shape (co)limits defined in `CategoryTheory.Limits.Types` are intended for use through the limits API, and the actual implementation should mostly be considered "sealed". In this file, we provide definitions of the "standard" special shapes of limits in `Type`, giving the expected definitional implementation: * the terminal object is `PUnit` * the binary product of `X` and `Y` is `X × Y` * the product of a family `f : J → Type` is `Π j, f j` * the coproduct of a family `f : J → Type` is `Σ j, f j` * the binary coproduct of `X` and `Y` is the sum type `X ⊕ Y` * the equalizer of a pair of maps `(g, h)` is the subtype `{x : Y // g x = h x}` * the coequalizer of a pair of maps `(f, g)` is the quotient of `Y` by `∀ x : Y, f x ~ g x` * the pullback of `f : X ⟶ Z` and `g : Y ⟶ Z` is the subtype `{ p : X × Y // f p.1 = g p.2 }` of the product We first construct terms of `IsLimit` and `LimitCone`, and then provide isomorphisms with the types generated by the `HasLimit` API. As an example, when setting up the monoidal category structure on `Type` we use the `Types.terminalLimitCone` and `Types.binaryProductLimitCone` definitions. -/ universe v u open CategoryTheory Limits namespace CategoryTheory.Limits.Types example : HasProducts.{v} (Type v) := inferInstance example [UnivLE.{v, u}] : HasProducts.{v} (Type u) := inferInstance -- This shortcut instance is required in `Mathlib.CategoryTheory.Closed.Types`, -- although I don't understand why, and wish it wasn't. instance : HasProducts.{v} (Type v) := inferInstance /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`. -/ @[simp 1001] theorem pi_lift_π_apply {β : Type v} [Small.{u} β] (f : β → Type u) {P : Type u} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := congr_fun (limit.lift_π (Fan.mk P s) ⟨b⟩) x #align category_theory.limits.types.pi_lift_π_apply CategoryTheory.Limits.Types.pi_lift_π_apply /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`, with specialized universes. -/ theorem pi_lift_π_apply' {β : Type v} (f : β → Type v) {P : Type v} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := by simp #align category_theory.limits.types.pi_lift_π_apply' CategoryTheory.Limits.Types.pi_lift_π_apply' /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`. -/ @[simp 1001] theorem pi_map_π_apply {β : Type v} [Small.{u} β] {f g : β → Type u} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := Limit.map_π_apply.{v, u} _ _ _ #align category_theory.limits.types.pi_map_π_apply CategoryTheory.Limits.Types.pi_map_π_apply /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`, with specialized universes. -/ theorem pi_map_π_apply' {β : Type v} {f g : β → Type v} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := by simp #align category_theory.limits.types.pi_map_π_apply' CategoryTheory.Limits.Types.pi_map_π_apply' /-- The category of types has `PUnit` as a terminal object. -/ def terminalLimitCone : Limits.LimitCone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cone := { pt := PUnit π := (Functor.uniqueFromEmpty _).hom } isLimit := { lift := fun _ _ => PUnit.unit fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext apply Subsingleton.elim } #align category_theory.limits.types.terminal_limit_cone CategoryTheory.Limits.Types.terminalLimitCone /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def terminalIso : ⊤_ Type u ≅ PUnit := limit.isoLimitCone terminalLimitCone.{u, 0} #align category_theory.limits.types.terminal_iso CategoryTheory.Limits.Types.terminalIso /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def isTerminalPunit : IsTerminal (PUnit : Type u) := terminalIsTerminal.ofIso terminalIso #align category_theory.limits.types.is_terminal_punit CategoryTheory.Limits.Types.isTerminalPunit -- porting note: the following three instances have been added to ease -- the automation in a definition in `AlgebraicTopology.SimplicialSet` noncomputable instance : Inhabited (⊤_ (Type u)) := ⟨@terminal.from (Type u) _ _ (ULift (Fin 1)) (ULift.up 0)⟩ instance : Subsingleton (⊤_ (Type u)) := ⟨fun a b => congr_fun (@Subsingleton.elim (_ ⟶ ⊤_ (Type u)) _ (fun _ => a) (fun _ => b)) (ULift.up (0 : Fin 1))⟩ noncomputable instance : Unique (⊤_ (Type u)) := Unique.mk' _ /-- A type is terminal if and only if it contains exactly one element. -/ noncomputable def isTerminalEquivUnique (X : Type u) : IsTerminal X ≃ Unique X := equivOfSubsingletonOfSubsingleton (fun h => ((Iso.toEquiv (terminalIsoIsTerminal h).symm).unique)) (fun _ => IsTerminal.ofIso terminalIsTerminal (Equiv.toIso (Equiv.equivOfUnique _ _))) /-- A type is terminal if and only if it is isomorphic to `PUnit`. -/ noncomputable def isTerminalEquivIsoPUnit (X : Type u) : IsTerminal X ≃ (X ≅ PUnit) := by calc IsTerminal X ≃ Unique X := isTerminalEquivUnique _ _ ≃ (X ≃ PUnit.{u + 1}) := uniqueEquivEquivUnique _ _ _ ≃ (X ≅ PUnit) := equivEquivIso /-- The category of types has `PEmpty` as an initial object. -/ def initialColimitCocone : Limits.ColimitCocone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cocone := { pt := PEmpty ι := (Functor.uniqueFromEmpty _).inv } isColimit := { desc := fun _ => by rintro ⟨⟩ fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext x; cases x } #align category_theory.limits.types.initial_colimit_cocone CategoryTheory.Limits.Types.initialColimitCocone /-- The initial object in `Type u` is `PEmpty`. -/ noncomputable def initialIso : ⊥_ Type u ≅ PEmpty := colimit.isoColimitCocone initialColimitCocone.{u, 0} #align category_theory.limits.types.initial_iso CategoryTheory.Limits.Types.initialIso /-- The initial object in `Type u` is `PEmpty`. -/ noncomputable def isInitialPunit : IsInitial (PEmpty : Type u) := initialIsInitial.ofIso initialIso #align category_theory.limits.types.is_initial_punit CategoryTheory.Limits.Types.isInitialPunit open CategoryTheory.Limits.WalkingPair -- We manually generate the other projection lemmas since the simp-normal form for the legs is -- otherwise not created correctly. /-- The product type `X × Y` forms a cone for the binary product of `X` and `Y`. -/ @[simps! pt] def binaryProductCone (X Y : Type u) : BinaryFan X Y := BinaryFan.mk _root_.Prod.fst _root_.Prod.snd #align category_theory.limits.types.binary_product_cone CategoryTheory.Limits.Types.binaryProductCone @[simp] theorem binaryProductCone_fst (X Y : Type u) : (binaryProductCone X Y).fst = _root_.Prod.fst := rfl #align category_theory.limits.types.binary_product_cone_fst CategoryTheory.Limits.Types.binaryProductCone_fst @[simp] theorem binaryProductCone_snd (X Y : Type u) : (binaryProductCone X Y).snd = _root_.Prod.snd := rfl #align category_theory.limits.types.binary_product_cone_snd CategoryTheory.Limits.Types.binaryProductCone_snd /-- The product type `X × Y` is a binary product for `X` and `Y`. -/ @[simps] def binaryProductLimit (X Y : Type u) : IsLimit (binaryProductCone X Y) where lift (s : BinaryFan X Y) x := (s.fst x, s.snd x) fac _ j := Discrete.recOn j fun j => WalkingPair.casesOn j rfl rfl uniq _ _ w := funext fun x => Prod.ext (congr_fun (w ⟨left⟩) x) (congr_fun (w ⟨right⟩) x) #align category_theory.limits.types.binary_product_limit CategoryTheory.Limits.Types.binaryProductLimit /-- The category of types has `X × Y`, the usual cartesian product, as the binary product of `X` and `Y`. -/ @[simps] def binaryProductLimitCone (X Y : Type u) : Limits.LimitCone (pair X Y) := ⟨_, binaryProductLimit X Y⟩ #align category_theory.limits.types.binary_product_limit_cone CategoryTheory.Limits.Types.binaryProductLimitCone /-- The categorical binary product in `Type u` is cartesian product. -/ noncomputable def binaryProductIso (X Y : Type u) : Limits.prod X Y ≅ X × Y := limit.isoLimitCone (binaryProductLimitCone X Y) #align category_theory.limits.types.binary_product_iso CategoryTheory.Limits.Types.binaryProductIso @[elementwise (attr := simp)] theorem binaryProductIso_hom_comp_fst (X Y : Type u) : (binaryProductIso X Y).hom ≫ _root_.Prod.fst = Limits.prod.fst := limit.isoLimitCone_hom_π (binaryProductLimitCone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_product_iso_hom_comp_fst CategoryTheory.Limits.Types.binaryProductIso_hom_comp_fst @[elementwise (attr := simp)] theorem binaryProductIso_hom_comp_snd (X Y : Type u) : (binaryProductIso X Y).hom ≫ _root_.Prod.snd = Limits.prod.snd := limit.isoLimitCone_hom_π (binaryProductLimitCone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_product_iso_hom_comp_snd CategoryTheory.Limits.Types.binaryProductIso_hom_comp_snd @[elementwise (attr := simp)] theorem binaryProductIso_inv_comp_fst (X Y : Type u) : (binaryProductIso X Y).inv ≫ Limits.prod.fst = _root_.Prod.fst := limit.isoLimitCone_inv_π (binaryProductLimitCone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_product_iso_inv_comp_fst CategoryTheory.Limits.Types.binaryProductIso_inv_comp_fst @[elementwise (attr := simp)] theorem binaryProductIso_inv_comp_snd (X Y : Type u) : (binaryProductIso X Y).inv ≫ Limits.prod.snd = _root_.Prod.snd := limit.isoLimitCone_inv_π (binaryProductLimitCone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_product_iso_inv_comp_snd CategoryTheory.Limits.Types.binaryProductIso_inv_comp_snd -- porting note: it was originally @[simps (config := { typeMd := reducible })] -- We add the option `type_md` to tell `@[simps]` to not treat homomorphisms `X ⟶ Y` in `Type*` as -- a function type /-- The functor which sends `X, Y` to the product type `X × Y`. -/ @[simps] def binaryProductFunctor : Type u ⥤ Type u ⥤ Type u where obj X := { obj := fun Y => X × Y map := fun { Y₁ Y₂} f => (binaryProductLimit X Y₂).lift (BinaryFan.mk _root_.Prod.fst (_root_.Prod.snd ≫ f)) } map {X₁ X₂} f := { app := fun Y => (binaryProductLimit X₂ Y).lift (BinaryFan.mk (_root_.Prod.fst ≫ f) _root_.Prod.snd) } #align category_theory.limits.types.binary_product_functor CategoryTheory.Limits.Types.binaryProductFunctor /-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _) := by refine' NatIso.ofComponents (fun X => _) (fun _ => _) · refine' NatIso.ofComponents (fun Y => _) (fun _ => _) · exact ((limit.isLimit _).conePointUniqueUpToIso (binaryProductLimit X Y)).symm · apply Limits.prod.hom_ext <;> simp <;> rfl · ext : 2 apply Limits.prod.hom_ext <;> simp <;> rfl #align category_theory.limits.types.binary_product_iso_prod CategoryTheory.Limits.Types.binaryProductIsoProd /-- The sum type `X ⊕ Y` forms a cocone for the binary coproduct of `X` and `Y`. -/ @[simps!] def binaryCoproductCocone (X Y : Type u) : Cocone (pair X Y) := BinaryCofan.mk Sum.inl Sum.inr #align category_theory.limits.types.binary_coproduct_cocone CategoryTheory.Limits.Types.binaryCoproductCocone /-- The sum type `X ⊕ Y` is a binary coproduct for `X` and `Y`. -/ @[simps] def binaryCoproductColimit (X Y : Type u) : IsColimit (binaryCoproductCocone X Y) where desc := fun s : BinaryCofan X Y => Sum.elim s.inl s.inr fac _ j := Discrete.recOn j fun j => WalkingPair.casesOn j rfl rfl uniq _ _ w := funext fun x => Sum.casesOn x (congr_fun (w ⟨left⟩)) (congr_fun (w ⟨right⟩)) #align category_theory.limits.types.binary_coproduct_colimit CategoryTheory.Limits.Types.binaryCoproductColimit /-- The category of types has `X ⊕ Y`, as the binary coproduct of `X` and `Y`. -/ def binaryCoproductColimitCocone (X Y : Type u) : Limits.ColimitCocone (pair X Y) := ⟨_, binaryCoproductColimit X Y⟩ #align category_theory.limits.types.binary_coproduct_colimit_cocone CategoryTheory.Limits.Types.binaryCoproductColimitCocone /-- The categorical binary coproduct in `Type u` is the sum `X ⊕ Y`. -/ noncomputable def binaryCoproductIso (X Y : Type u) : Limits.coprod X Y ≅ Sum X Y := colimit.isoColimitCocone (binaryCoproductColimitCocone X Y) #align category_theory.limits.types.binary_coproduct_iso CategoryTheory.Limits.Types.binaryCoproductIso --open CategoryTheory.Type @[elementwise (attr := simp)] theorem binaryCoproductIso_inl_comp_hom (X Y : Type u) : Limits.coprod.inl ≫ (binaryCoproductIso X Y).hom = Sum.inl := colimit.isoColimitCocone_ι_hom (binaryCoproductColimitCocone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_coproduct_iso_inl_comp_hom CategoryTheory.Limits.Types.binaryCoproductIso_inl_comp_hom @[elementwise (attr := simp)] theorem binaryCoproductIso_inr_comp_hom (X Y : Type u) : Limits.coprod.inr ≫ (binaryCoproductIso X Y).hom = Sum.inr := colimit.isoColimitCocone_ι_hom (binaryCoproductColimitCocone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_coproduct_iso_inr_comp_hom CategoryTheory.Limits.Types.binaryCoproductIso_inr_comp_hom @[elementwise (attr := simp)] theorem binaryCoproductIso_inl_comp_inv (X Y : Type u) : ↾(Sum.inl : X ⟶ Sum X Y) ≫ (binaryCoproductIso X Y).inv = Limits.coprod.inl := colimit.isoColimitCocone_ι_inv (binaryCoproductColimitCocone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_coproduct_iso_inl_comp_inv CategoryTheory.Limits.Types.binaryCoproductIso_inl_comp_inv @[elementwise (attr := simp)] theorem binaryCoproductIso_inr_comp_inv (X Y : Type u) : ↾(Sum.inr : Y ⟶ Sum X Y) ≫ (binaryCoproductIso X Y).inv = Limits.coprod.inr := colimit.isoColimitCocone_ι_inv (binaryCoproductColimitCocone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_coproduct_iso_inr_comp_inv CategoryTheory.Limits.Types.binaryCoproductIso_inr_comp_inv open Function (Injective) theorem binaryCofan_isColimit_iff {X Y : Type u} (c : BinaryCofan X Y) : Nonempty (IsColimit c) ↔ Injective c.inl ∧ Injective c.inr ∧ IsCompl (Set.range c.inl) (Set.range c.inr) := by classical constructor · rintro ⟨h⟩ rw [← show _ = c.inl from h.comp_coconePointUniqueUpToIso_inv (binaryCoproductColimit X Y) ⟨WalkingPair.left⟩, ← show _ = c.inr from h.comp_coconePointUniqueUpToIso_inv (binaryCoproductColimit X Y) ⟨WalkingPair.right⟩] dsimp [binaryCoproductCocone]
refine' ⟨(h.coconePointUniqueUpToIso (binaryCoproductColimit X Y)).symm.toEquiv.injective.comp Sum.inl_injective, (h.coconePointUniqueUpToIso (binaryCoproductColimit X Y)).symm.toEquiv.injective.comp Sum.inr_injective, _⟩
theorem binaryCofan_isColimit_iff {X Y : Type u} (c : BinaryCofan X Y) : Nonempty (IsColimit c) ↔ Injective c.inl ∧ Injective c.inr ∧ IsCompl (Set.range c.inl) (Set.range c.inr) := by classical constructor · rintro ⟨h⟩ rw [← show _ = c.inl from h.comp_coconePointUniqueUpToIso_inv (binaryCoproductColimit X Y) ⟨WalkingPair.left⟩, ← show _ = c.inr from h.comp_coconePointUniqueUpToIso_inv (binaryCoproductColimit X Y) ⟨WalkingPair.right⟩] dsimp [binaryCoproductCocone]
Mathlib.CategoryTheory.Limits.Shapes.Types.302_0.ctQAUYXLRXnvMGw
theorem binaryCofan_isColimit_iff {X Y : Type u} (c : BinaryCofan X Y) : Nonempty (IsColimit c) ↔ Injective c.inl ∧ Injective c.inr ∧ IsCompl (Set.range c.inl) (Set.range c.inr)
Mathlib_CategoryTheory_Limits_Shapes_Types
case mp.intro X Y : Type u c : BinaryCofan X Y h : IsColimit c ⊢ IsCompl (Set.range (Sum.inl ≫ (IsColimit.coconePointUniqueUpToIso h (binaryCoproductColimit X Y)).inv)) (Set.range (Sum.inr ≫ (IsColimit.coconePointUniqueUpToIso h (binaryCoproductColimit X Y)).inv))
/- Copyright (c) 2020 Scott Morrison. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Scott Morrison -/ import Mathlib.CategoryTheory.Limits.Types import Mathlib.CategoryTheory.Limits.Shapes.Products import Mathlib.CategoryTheory.Limits.Shapes.BinaryProducts import Mathlib.CategoryTheory.Limits.Shapes.Terminal import Mathlib.CategoryTheory.ConcreteCategory.Basic import Mathlib.Tactic.CategoryTheory.Elementwise #align_import category_theory.limits.shapes.types from "leanprover-community/mathlib"@"5dc6092d09e5e489106865241986f7f2ad28d4c8" /-! # Special shapes for limits in `Type`. The general shape (co)limits defined in `CategoryTheory.Limits.Types` are intended for use through the limits API, and the actual implementation should mostly be considered "sealed". In this file, we provide definitions of the "standard" special shapes of limits in `Type`, giving the expected definitional implementation: * the terminal object is `PUnit` * the binary product of `X` and `Y` is `X × Y` * the product of a family `f : J → Type` is `Π j, f j` * the coproduct of a family `f : J → Type` is `Σ j, f j` * the binary coproduct of `X` and `Y` is the sum type `X ⊕ Y` * the equalizer of a pair of maps `(g, h)` is the subtype `{x : Y // g x = h x}` * the coequalizer of a pair of maps `(f, g)` is the quotient of `Y` by `∀ x : Y, f x ~ g x` * the pullback of `f : X ⟶ Z` and `g : Y ⟶ Z` is the subtype `{ p : X × Y // f p.1 = g p.2 }` of the product We first construct terms of `IsLimit` and `LimitCone`, and then provide isomorphisms with the types generated by the `HasLimit` API. As an example, when setting up the monoidal category structure on `Type` we use the `Types.terminalLimitCone` and `Types.binaryProductLimitCone` definitions. -/ universe v u open CategoryTheory Limits namespace CategoryTheory.Limits.Types example : HasProducts.{v} (Type v) := inferInstance example [UnivLE.{v, u}] : HasProducts.{v} (Type u) := inferInstance -- This shortcut instance is required in `Mathlib.CategoryTheory.Closed.Types`, -- although I don't understand why, and wish it wasn't. instance : HasProducts.{v} (Type v) := inferInstance /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`. -/ @[simp 1001] theorem pi_lift_π_apply {β : Type v} [Small.{u} β] (f : β → Type u) {P : Type u} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := congr_fun (limit.lift_π (Fan.mk P s) ⟨b⟩) x #align category_theory.limits.types.pi_lift_π_apply CategoryTheory.Limits.Types.pi_lift_π_apply /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`, with specialized universes. -/ theorem pi_lift_π_apply' {β : Type v} (f : β → Type v) {P : Type v} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := by simp #align category_theory.limits.types.pi_lift_π_apply' CategoryTheory.Limits.Types.pi_lift_π_apply' /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`. -/ @[simp 1001] theorem pi_map_π_apply {β : Type v} [Small.{u} β] {f g : β → Type u} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := Limit.map_π_apply.{v, u} _ _ _ #align category_theory.limits.types.pi_map_π_apply CategoryTheory.Limits.Types.pi_map_π_apply /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`, with specialized universes. -/ theorem pi_map_π_apply' {β : Type v} {f g : β → Type v} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := by simp #align category_theory.limits.types.pi_map_π_apply' CategoryTheory.Limits.Types.pi_map_π_apply' /-- The category of types has `PUnit` as a terminal object. -/ def terminalLimitCone : Limits.LimitCone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cone := { pt := PUnit π := (Functor.uniqueFromEmpty _).hom } isLimit := { lift := fun _ _ => PUnit.unit fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext apply Subsingleton.elim } #align category_theory.limits.types.terminal_limit_cone CategoryTheory.Limits.Types.terminalLimitCone /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def terminalIso : ⊤_ Type u ≅ PUnit := limit.isoLimitCone terminalLimitCone.{u, 0} #align category_theory.limits.types.terminal_iso CategoryTheory.Limits.Types.terminalIso /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def isTerminalPunit : IsTerminal (PUnit : Type u) := terminalIsTerminal.ofIso terminalIso #align category_theory.limits.types.is_terminal_punit CategoryTheory.Limits.Types.isTerminalPunit -- porting note: the following three instances have been added to ease -- the automation in a definition in `AlgebraicTopology.SimplicialSet` noncomputable instance : Inhabited (⊤_ (Type u)) := ⟨@terminal.from (Type u) _ _ (ULift (Fin 1)) (ULift.up 0)⟩ instance : Subsingleton (⊤_ (Type u)) := ⟨fun a b => congr_fun (@Subsingleton.elim (_ ⟶ ⊤_ (Type u)) _ (fun _ => a) (fun _ => b)) (ULift.up (0 : Fin 1))⟩ noncomputable instance : Unique (⊤_ (Type u)) := Unique.mk' _ /-- A type is terminal if and only if it contains exactly one element. -/ noncomputable def isTerminalEquivUnique (X : Type u) : IsTerminal X ≃ Unique X := equivOfSubsingletonOfSubsingleton (fun h => ((Iso.toEquiv (terminalIsoIsTerminal h).symm).unique)) (fun _ => IsTerminal.ofIso terminalIsTerminal (Equiv.toIso (Equiv.equivOfUnique _ _))) /-- A type is terminal if and only if it is isomorphic to `PUnit`. -/ noncomputable def isTerminalEquivIsoPUnit (X : Type u) : IsTerminal X ≃ (X ≅ PUnit) := by calc IsTerminal X ≃ Unique X := isTerminalEquivUnique _ _ ≃ (X ≃ PUnit.{u + 1}) := uniqueEquivEquivUnique _ _ _ ≃ (X ≅ PUnit) := equivEquivIso /-- The category of types has `PEmpty` as an initial object. -/ def initialColimitCocone : Limits.ColimitCocone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cocone := { pt := PEmpty ι := (Functor.uniqueFromEmpty _).inv } isColimit := { desc := fun _ => by rintro ⟨⟩ fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext x; cases x } #align category_theory.limits.types.initial_colimit_cocone CategoryTheory.Limits.Types.initialColimitCocone /-- The initial object in `Type u` is `PEmpty`. -/ noncomputable def initialIso : ⊥_ Type u ≅ PEmpty := colimit.isoColimitCocone initialColimitCocone.{u, 0} #align category_theory.limits.types.initial_iso CategoryTheory.Limits.Types.initialIso /-- The initial object in `Type u` is `PEmpty`. -/ noncomputable def isInitialPunit : IsInitial (PEmpty : Type u) := initialIsInitial.ofIso initialIso #align category_theory.limits.types.is_initial_punit CategoryTheory.Limits.Types.isInitialPunit open CategoryTheory.Limits.WalkingPair -- We manually generate the other projection lemmas since the simp-normal form for the legs is -- otherwise not created correctly. /-- The product type `X × Y` forms a cone for the binary product of `X` and `Y`. -/ @[simps! pt] def binaryProductCone (X Y : Type u) : BinaryFan X Y := BinaryFan.mk _root_.Prod.fst _root_.Prod.snd #align category_theory.limits.types.binary_product_cone CategoryTheory.Limits.Types.binaryProductCone @[simp] theorem binaryProductCone_fst (X Y : Type u) : (binaryProductCone X Y).fst = _root_.Prod.fst := rfl #align category_theory.limits.types.binary_product_cone_fst CategoryTheory.Limits.Types.binaryProductCone_fst @[simp] theorem binaryProductCone_snd (X Y : Type u) : (binaryProductCone X Y).snd = _root_.Prod.snd := rfl #align category_theory.limits.types.binary_product_cone_snd CategoryTheory.Limits.Types.binaryProductCone_snd /-- The product type `X × Y` is a binary product for `X` and `Y`. -/ @[simps] def binaryProductLimit (X Y : Type u) : IsLimit (binaryProductCone X Y) where lift (s : BinaryFan X Y) x := (s.fst x, s.snd x) fac _ j := Discrete.recOn j fun j => WalkingPair.casesOn j rfl rfl uniq _ _ w := funext fun x => Prod.ext (congr_fun (w ⟨left⟩) x) (congr_fun (w ⟨right⟩) x) #align category_theory.limits.types.binary_product_limit CategoryTheory.Limits.Types.binaryProductLimit /-- The category of types has `X × Y`, the usual cartesian product, as the binary product of `X` and `Y`. -/ @[simps] def binaryProductLimitCone (X Y : Type u) : Limits.LimitCone (pair X Y) := ⟨_, binaryProductLimit X Y⟩ #align category_theory.limits.types.binary_product_limit_cone CategoryTheory.Limits.Types.binaryProductLimitCone /-- The categorical binary product in `Type u` is cartesian product. -/ noncomputable def binaryProductIso (X Y : Type u) : Limits.prod X Y ≅ X × Y := limit.isoLimitCone (binaryProductLimitCone X Y) #align category_theory.limits.types.binary_product_iso CategoryTheory.Limits.Types.binaryProductIso @[elementwise (attr := simp)] theorem binaryProductIso_hom_comp_fst (X Y : Type u) : (binaryProductIso X Y).hom ≫ _root_.Prod.fst = Limits.prod.fst := limit.isoLimitCone_hom_π (binaryProductLimitCone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_product_iso_hom_comp_fst CategoryTheory.Limits.Types.binaryProductIso_hom_comp_fst @[elementwise (attr := simp)] theorem binaryProductIso_hom_comp_snd (X Y : Type u) : (binaryProductIso X Y).hom ≫ _root_.Prod.snd = Limits.prod.snd := limit.isoLimitCone_hom_π (binaryProductLimitCone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_product_iso_hom_comp_snd CategoryTheory.Limits.Types.binaryProductIso_hom_comp_snd @[elementwise (attr := simp)] theorem binaryProductIso_inv_comp_fst (X Y : Type u) : (binaryProductIso X Y).inv ≫ Limits.prod.fst = _root_.Prod.fst := limit.isoLimitCone_inv_π (binaryProductLimitCone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_product_iso_inv_comp_fst CategoryTheory.Limits.Types.binaryProductIso_inv_comp_fst @[elementwise (attr := simp)] theorem binaryProductIso_inv_comp_snd (X Y : Type u) : (binaryProductIso X Y).inv ≫ Limits.prod.snd = _root_.Prod.snd := limit.isoLimitCone_inv_π (binaryProductLimitCone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_product_iso_inv_comp_snd CategoryTheory.Limits.Types.binaryProductIso_inv_comp_snd -- porting note: it was originally @[simps (config := { typeMd := reducible })] -- We add the option `type_md` to tell `@[simps]` to not treat homomorphisms `X ⟶ Y` in `Type*` as -- a function type /-- The functor which sends `X, Y` to the product type `X × Y`. -/ @[simps] def binaryProductFunctor : Type u ⥤ Type u ⥤ Type u where obj X := { obj := fun Y => X × Y map := fun { Y₁ Y₂} f => (binaryProductLimit X Y₂).lift (BinaryFan.mk _root_.Prod.fst (_root_.Prod.snd ≫ f)) } map {X₁ X₂} f := { app := fun Y => (binaryProductLimit X₂ Y).lift (BinaryFan.mk (_root_.Prod.fst ≫ f) _root_.Prod.snd) } #align category_theory.limits.types.binary_product_functor CategoryTheory.Limits.Types.binaryProductFunctor /-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _) := by refine' NatIso.ofComponents (fun X => _) (fun _ => _) · refine' NatIso.ofComponents (fun Y => _) (fun _ => _) · exact ((limit.isLimit _).conePointUniqueUpToIso (binaryProductLimit X Y)).symm · apply Limits.prod.hom_ext <;> simp <;> rfl · ext : 2 apply Limits.prod.hom_ext <;> simp <;> rfl #align category_theory.limits.types.binary_product_iso_prod CategoryTheory.Limits.Types.binaryProductIsoProd /-- The sum type `X ⊕ Y` forms a cocone for the binary coproduct of `X` and `Y`. -/ @[simps!] def binaryCoproductCocone (X Y : Type u) : Cocone (pair X Y) := BinaryCofan.mk Sum.inl Sum.inr #align category_theory.limits.types.binary_coproduct_cocone CategoryTheory.Limits.Types.binaryCoproductCocone /-- The sum type `X ⊕ Y` is a binary coproduct for `X` and `Y`. -/ @[simps] def binaryCoproductColimit (X Y : Type u) : IsColimit (binaryCoproductCocone X Y) where desc := fun s : BinaryCofan X Y => Sum.elim s.inl s.inr fac _ j := Discrete.recOn j fun j => WalkingPair.casesOn j rfl rfl uniq _ _ w := funext fun x => Sum.casesOn x (congr_fun (w ⟨left⟩)) (congr_fun (w ⟨right⟩)) #align category_theory.limits.types.binary_coproduct_colimit CategoryTheory.Limits.Types.binaryCoproductColimit /-- The category of types has `X ⊕ Y`, as the binary coproduct of `X` and `Y`. -/ def binaryCoproductColimitCocone (X Y : Type u) : Limits.ColimitCocone (pair X Y) := ⟨_, binaryCoproductColimit X Y⟩ #align category_theory.limits.types.binary_coproduct_colimit_cocone CategoryTheory.Limits.Types.binaryCoproductColimitCocone /-- The categorical binary coproduct in `Type u` is the sum `X ⊕ Y`. -/ noncomputable def binaryCoproductIso (X Y : Type u) : Limits.coprod X Y ≅ Sum X Y := colimit.isoColimitCocone (binaryCoproductColimitCocone X Y) #align category_theory.limits.types.binary_coproduct_iso CategoryTheory.Limits.Types.binaryCoproductIso --open CategoryTheory.Type @[elementwise (attr := simp)] theorem binaryCoproductIso_inl_comp_hom (X Y : Type u) : Limits.coprod.inl ≫ (binaryCoproductIso X Y).hom = Sum.inl := colimit.isoColimitCocone_ι_hom (binaryCoproductColimitCocone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_coproduct_iso_inl_comp_hom CategoryTheory.Limits.Types.binaryCoproductIso_inl_comp_hom @[elementwise (attr := simp)] theorem binaryCoproductIso_inr_comp_hom (X Y : Type u) : Limits.coprod.inr ≫ (binaryCoproductIso X Y).hom = Sum.inr := colimit.isoColimitCocone_ι_hom (binaryCoproductColimitCocone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_coproduct_iso_inr_comp_hom CategoryTheory.Limits.Types.binaryCoproductIso_inr_comp_hom @[elementwise (attr := simp)] theorem binaryCoproductIso_inl_comp_inv (X Y : Type u) : ↾(Sum.inl : X ⟶ Sum X Y) ≫ (binaryCoproductIso X Y).inv = Limits.coprod.inl := colimit.isoColimitCocone_ι_inv (binaryCoproductColimitCocone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_coproduct_iso_inl_comp_inv CategoryTheory.Limits.Types.binaryCoproductIso_inl_comp_inv @[elementwise (attr := simp)] theorem binaryCoproductIso_inr_comp_inv (X Y : Type u) : ↾(Sum.inr : Y ⟶ Sum X Y) ≫ (binaryCoproductIso X Y).inv = Limits.coprod.inr := colimit.isoColimitCocone_ι_inv (binaryCoproductColimitCocone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_coproduct_iso_inr_comp_inv CategoryTheory.Limits.Types.binaryCoproductIso_inr_comp_inv open Function (Injective) theorem binaryCofan_isColimit_iff {X Y : Type u} (c : BinaryCofan X Y) : Nonempty (IsColimit c) ↔ Injective c.inl ∧ Injective c.inr ∧ IsCompl (Set.range c.inl) (Set.range c.inr) := by classical constructor · rintro ⟨h⟩ rw [← show _ = c.inl from h.comp_coconePointUniqueUpToIso_inv (binaryCoproductColimit X Y) ⟨WalkingPair.left⟩, ← show _ = c.inr from h.comp_coconePointUniqueUpToIso_inv (binaryCoproductColimit X Y) ⟨WalkingPair.right⟩] dsimp [binaryCoproductCocone] refine' ⟨(h.coconePointUniqueUpToIso (binaryCoproductColimit X Y)).symm.toEquiv.injective.comp Sum.inl_injective, (h.coconePointUniqueUpToIso (binaryCoproductColimit X Y)).symm.toEquiv.injective.comp Sum.inr_injective, _⟩
erw [Set.range_comp, ← eq_compl_iff_isCompl, Set.range_comp _ Sum.inr, ← Set.image_compl_eq (h.coconePointUniqueUpToIso (binaryCoproductColimit X Y)).symm.toEquiv.bijective]
theorem binaryCofan_isColimit_iff {X Y : Type u} (c : BinaryCofan X Y) : Nonempty (IsColimit c) ↔ Injective c.inl ∧ Injective c.inr ∧ IsCompl (Set.range c.inl) (Set.range c.inr) := by classical constructor · rintro ⟨h⟩ rw [← show _ = c.inl from h.comp_coconePointUniqueUpToIso_inv (binaryCoproductColimit X Y) ⟨WalkingPair.left⟩, ← show _ = c.inr from h.comp_coconePointUniqueUpToIso_inv (binaryCoproductColimit X Y) ⟨WalkingPair.right⟩] dsimp [binaryCoproductCocone] refine' ⟨(h.coconePointUniqueUpToIso (binaryCoproductColimit X Y)).symm.toEquiv.injective.comp Sum.inl_injective, (h.coconePointUniqueUpToIso (binaryCoproductColimit X Y)).symm.toEquiv.injective.comp Sum.inr_injective, _⟩
Mathlib.CategoryTheory.Limits.Shapes.Types.302_0.ctQAUYXLRXnvMGw
theorem binaryCofan_isColimit_iff {X Y : Type u} (c : BinaryCofan X Y) : Nonempty (IsColimit c) ↔ Injective c.inl ∧ Injective c.inr ∧ IsCompl (Set.range c.inl) (Set.range c.inr)
Mathlib_CategoryTheory_Limits_Shapes_Types
case mp.intro X Y : Type u c : BinaryCofan X Y h : IsColimit c ⊢ (IsColimit.coconePointUniqueUpToIso h (binaryCoproductColimit X Y)).inv '' Set.range Sum.inl = ⇑(IsColimit.coconePointUniqueUpToIso h (binaryCoproductColimit X Y)).symm.toEquiv '' (Set.range Sum.inr)ᶜ
/- Copyright (c) 2020 Scott Morrison. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Scott Morrison -/ import Mathlib.CategoryTheory.Limits.Types import Mathlib.CategoryTheory.Limits.Shapes.Products import Mathlib.CategoryTheory.Limits.Shapes.BinaryProducts import Mathlib.CategoryTheory.Limits.Shapes.Terminal import Mathlib.CategoryTheory.ConcreteCategory.Basic import Mathlib.Tactic.CategoryTheory.Elementwise #align_import category_theory.limits.shapes.types from "leanprover-community/mathlib"@"5dc6092d09e5e489106865241986f7f2ad28d4c8" /-! # Special shapes for limits in `Type`. The general shape (co)limits defined in `CategoryTheory.Limits.Types` are intended for use through the limits API, and the actual implementation should mostly be considered "sealed". In this file, we provide definitions of the "standard" special shapes of limits in `Type`, giving the expected definitional implementation: * the terminal object is `PUnit` * the binary product of `X` and `Y` is `X × Y` * the product of a family `f : J → Type` is `Π j, f j` * the coproduct of a family `f : J → Type` is `Σ j, f j` * the binary coproduct of `X` and `Y` is the sum type `X ⊕ Y` * the equalizer of a pair of maps `(g, h)` is the subtype `{x : Y // g x = h x}` * the coequalizer of a pair of maps `(f, g)` is the quotient of `Y` by `∀ x : Y, f x ~ g x` * the pullback of `f : X ⟶ Z` and `g : Y ⟶ Z` is the subtype `{ p : X × Y // f p.1 = g p.2 }` of the product We first construct terms of `IsLimit` and `LimitCone`, and then provide isomorphisms with the types generated by the `HasLimit` API. As an example, when setting up the monoidal category structure on `Type` we use the `Types.terminalLimitCone` and `Types.binaryProductLimitCone` definitions. -/ universe v u open CategoryTheory Limits namespace CategoryTheory.Limits.Types example : HasProducts.{v} (Type v) := inferInstance example [UnivLE.{v, u}] : HasProducts.{v} (Type u) := inferInstance -- This shortcut instance is required in `Mathlib.CategoryTheory.Closed.Types`, -- although I don't understand why, and wish it wasn't. instance : HasProducts.{v} (Type v) := inferInstance /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`. -/ @[simp 1001] theorem pi_lift_π_apply {β : Type v} [Small.{u} β] (f : β → Type u) {P : Type u} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := congr_fun (limit.lift_π (Fan.mk P s) ⟨b⟩) x #align category_theory.limits.types.pi_lift_π_apply CategoryTheory.Limits.Types.pi_lift_π_apply /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`, with specialized universes. -/ theorem pi_lift_π_apply' {β : Type v} (f : β → Type v) {P : Type v} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := by simp #align category_theory.limits.types.pi_lift_π_apply' CategoryTheory.Limits.Types.pi_lift_π_apply' /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`. -/ @[simp 1001] theorem pi_map_π_apply {β : Type v} [Small.{u} β] {f g : β → Type u} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := Limit.map_π_apply.{v, u} _ _ _ #align category_theory.limits.types.pi_map_π_apply CategoryTheory.Limits.Types.pi_map_π_apply /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`, with specialized universes. -/ theorem pi_map_π_apply' {β : Type v} {f g : β → Type v} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := by simp #align category_theory.limits.types.pi_map_π_apply' CategoryTheory.Limits.Types.pi_map_π_apply' /-- The category of types has `PUnit` as a terminal object. -/ def terminalLimitCone : Limits.LimitCone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cone := { pt := PUnit π := (Functor.uniqueFromEmpty _).hom } isLimit := { lift := fun _ _ => PUnit.unit fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext apply Subsingleton.elim } #align category_theory.limits.types.terminal_limit_cone CategoryTheory.Limits.Types.terminalLimitCone /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def terminalIso : ⊤_ Type u ≅ PUnit := limit.isoLimitCone terminalLimitCone.{u, 0} #align category_theory.limits.types.terminal_iso CategoryTheory.Limits.Types.terminalIso /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def isTerminalPunit : IsTerminal (PUnit : Type u) := terminalIsTerminal.ofIso terminalIso #align category_theory.limits.types.is_terminal_punit CategoryTheory.Limits.Types.isTerminalPunit -- porting note: the following three instances have been added to ease -- the automation in a definition in `AlgebraicTopology.SimplicialSet` noncomputable instance : Inhabited (⊤_ (Type u)) := ⟨@terminal.from (Type u) _ _ (ULift (Fin 1)) (ULift.up 0)⟩ instance : Subsingleton (⊤_ (Type u)) := ⟨fun a b => congr_fun (@Subsingleton.elim (_ ⟶ ⊤_ (Type u)) _ (fun _ => a) (fun _ => b)) (ULift.up (0 : Fin 1))⟩ noncomputable instance : Unique (⊤_ (Type u)) := Unique.mk' _ /-- A type is terminal if and only if it contains exactly one element. -/ noncomputable def isTerminalEquivUnique (X : Type u) : IsTerminal X ≃ Unique X := equivOfSubsingletonOfSubsingleton (fun h => ((Iso.toEquiv (terminalIsoIsTerminal h).symm).unique)) (fun _ => IsTerminal.ofIso terminalIsTerminal (Equiv.toIso (Equiv.equivOfUnique _ _))) /-- A type is terminal if and only if it is isomorphic to `PUnit`. -/ noncomputable def isTerminalEquivIsoPUnit (X : Type u) : IsTerminal X ≃ (X ≅ PUnit) := by calc IsTerminal X ≃ Unique X := isTerminalEquivUnique _ _ ≃ (X ≃ PUnit.{u + 1}) := uniqueEquivEquivUnique _ _ _ ≃ (X ≅ PUnit) := equivEquivIso /-- The category of types has `PEmpty` as an initial object. -/ def initialColimitCocone : Limits.ColimitCocone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cocone := { pt := PEmpty ι := (Functor.uniqueFromEmpty _).inv } isColimit := { desc := fun _ => by rintro ⟨⟩ fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext x; cases x } #align category_theory.limits.types.initial_colimit_cocone CategoryTheory.Limits.Types.initialColimitCocone /-- The initial object in `Type u` is `PEmpty`. -/ noncomputable def initialIso : ⊥_ Type u ≅ PEmpty := colimit.isoColimitCocone initialColimitCocone.{u, 0} #align category_theory.limits.types.initial_iso CategoryTheory.Limits.Types.initialIso /-- The initial object in `Type u` is `PEmpty`. -/ noncomputable def isInitialPunit : IsInitial (PEmpty : Type u) := initialIsInitial.ofIso initialIso #align category_theory.limits.types.is_initial_punit CategoryTheory.Limits.Types.isInitialPunit open CategoryTheory.Limits.WalkingPair -- We manually generate the other projection lemmas since the simp-normal form for the legs is -- otherwise not created correctly. /-- The product type `X × Y` forms a cone for the binary product of `X` and `Y`. -/ @[simps! pt] def binaryProductCone (X Y : Type u) : BinaryFan X Y := BinaryFan.mk _root_.Prod.fst _root_.Prod.snd #align category_theory.limits.types.binary_product_cone CategoryTheory.Limits.Types.binaryProductCone @[simp] theorem binaryProductCone_fst (X Y : Type u) : (binaryProductCone X Y).fst = _root_.Prod.fst := rfl #align category_theory.limits.types.binary_product_cone_fst CategoryTheory.Limits.Types.binaryProductCone_fst @[simp] theorem binaryProductCone_snd (X Y : Type u) : (binaryProductCone X Y).snd = _root_.Prod.snd := rfl #align category_theory.limits.types.binary_product_cone_snd CategoryTheory.Limits.Types.binaryProductCone_snd /-- The product type `X × Y` is a binary product for `X` and `Y`. -/ @[simps] def binaryProductLimit (X Y : Type u) : IsLimit (binaryProductCone X Y) where lift (s : BinaryFan X Y) x := (s.fst x, s.snd x) fac _ j := Discrete.recOn j fun j => WalkingPair.casesOn j rfl rfl uniq _ _ w := funext fun x => Prod.ext (congr_fun (w ⟨left⟩) x) (congr_fun (w ⟨right⟩) x) #align category_theory.limits.types.binary_product_limit CategoryTheory.Limits.Types.binaryProductLimit /-- The category of types has `X × Y`, the usual cartesian product, as the binary product of `X` and `Y`. -/ @[simps] def binaryProductLimitCone (X Y : Type u) : Limits.LimitCone (pair X Y) := ⟨_, binaryProductLimit X Y⟩ #align category_theory.limits.types.binary_product_limit_cone CategoryTheory.Limits.Types.binaryProductLimitCone /-- The categorical binary product in `Type u` is cartesian product. -/ noncomputable def binaryProductIso (X Y : Type u) : Limits.prod X Y ≅ X × Y := limit.isoLimitCone (binaryProductLimitCone X Y) #align category_theory.limits.types.binary_product_iso CategoryTheory.Limits.Types.binaryProductIso @[elementwise (attr := simp)] theorem binaryProductIso_hom_comp_fst (X Y : Type u) : (binaryProductIso X Y).hom ≫ _root_.Prod.fst = Limits.prod.fst := limit.isoLimitCone_hom_π (binaryProductLimitCone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_product_iso_hom_comp_fst CategoryTheory.Limits.Types.binaryProductIso_hom_comp_fst @[elementwise (attr := simp)] theorem binaryProductIso_hom_comp_snd (X Y : Type u) : (binaryProductIso X Y).hom ≫ _root_.Prod.snd = Limits.prod.snd := limit.isoLimitCone_hom_π (binaryProductLimitCone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_product_iso_hom_comp_snd CategoryTheory.Limits.Types.binaryProductIso_hom_comp_snd @[elementwise (attr := simp)] theorem binaryProductIso_inv_comp_fst (X Y : Type u) : (binaryProductIso X Y).inv ≫ Limits.prod.fst = _root_.Prod.fst := limit.isoLimitCone_inv_π (binaryProductLimitCone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_product_iso_inv_comp_fst CategoryTheory.Limits.Types.binaryProductIso_inv_comp_fst @[elementwise (attr := simp)] theorem binaryProductIso_inv_comp_snd (X Y : Type u) : (binaryProductIso X Y).inv ≫ Limits.prod.snd = _root_.Prod.snd := limit.isoLimitCone_inv_π (binaryProductLimitCone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_product_iso_inv_comp_snd CategoryTheory.Limits.Types.binaryProductIso_inv_comp_snd -- porting note: it was originally @[simps (config := { typeMd := reducible })] -- We add the option `type_md` to tell `@[simps]` to not treat homomorphisms `X ⟶ Y` in `Type*` as -- a function type /-- The functor which sends `X, Y` to the product type `X × Y`. -/ @[simps] def binaryProductFunctor : Type u ⥤ Type u ⥤ Type u where obj X := { obj := fun Y => X × Y map := fun { Y₁ Y₂} f => (binaryProductLimit X Y₂).lift (BinaryFan.mk _root_.Prod.fst (_root_.Prod.snd ≫ f)) } map {X₁ X₂} f := { app := fun Y => (binaryProductLimit X₂ Y).lift (BinaryFan.mk (_root_.Prod.fst ≫ f) _root_.Prod.snd) } #align category_theory.limits.types.binary_product_functor CategoryTheory.Limits.Types.binaryProductFunctor /-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _) := by refine' NatIso.ofComponents (fun X => _) (fun _ => _) · refine' NatIso.ofComponents (fun Y => _) (fun _ => _) · exact ((limit.isLimit _).conePointUniqueUpToIso (binaryProductLimit X Y)).symm · apply Limits.prod.hom_ext <;> simp <;> rfl · ext : 2 apply Limits.prod.hom_ext <;> simp <;> rfl #align category_theory.limits.types.binary_product_iso_prod CategoryTheory.Limits.Types.binaryProductIsoProd /-- The sum type `X ⊕ Y` forms a cocone for the binary coproduct of `X` and `Y`. -/ @[simps!] def binaryCoproductCocone (X Y : Type u) : Cocone (pair X Y) := BinaryCofan.mk Sum.inl Sum.inr #align category_theory.limits.types.binary_coproduct_cocone CategoryTheory.Limits.Types.binaryCoproductCocone /-- The sum type `X ⊕ Y` is a binary coproduct for `X` and `Y`. -/ @[simps] def binaryCoproductColimit (X Y : Type u) : IsColimit (binaryCoproductCocone X Y) where desc := fun s : BinaryCofan X Y => Sum.elim s.inl s.inr fac _ j := Discrete.recOn j fun j => WalkingPair.casesOn j rfl rfl uniq _ _ w := funext fun x => Sum.casesOn x (congr_fun (w ⟨left⟩)) (congr_fun (w ⟨right⟩)) #align category_theory.limits.types.binary_coproduct_colimit CategoryTheory.Limits.Types.binaryCoproductColimit /-- The category of types has `X ⊕ Y`, as the binary coproduct of `X` and `Y`. -/ def binaryCoproductColimitCocone (X Y : Type u) : Limits.ColimitCocone (pair X Y) := ⟨_, binaryCoproductColimit X Y⟩ #align category_theory.limits.types.binary_coproduct_colimit_cocone CategoryTheory.Limits.Types.binaryCoproductColimitCocone /-- The categorical binary coproduct in `Type u` is the sum `X ⊕ Y`. -/ noncomputable def binaryCoproductIso (X Y : Type u) : Limits.coprod X Y ≅ Sum X Y := colimit.isoColimitCocone (binaryCoproductColimitCocone X Y) #align category_theory.limits.types.binary_coproduct_iso CategoryTheory.Limits.Types.binaryCoproductIso --open CategoryTheory.Type @[elementwise (attr := simp)] theorem binaryCoproductIso_inl_comp_hom (X Y : Type u) : Limits.coprod.inl ≫ (binaryCoproductIso X Y).hom = Sum.inl := colimit.isoColimitCocone_ι_hom (binaryCoproductColimitCocone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_coproduct_iso_inl_comp_hom CategoryTheory.Limits.Types.binaryCoproductIso_inl_comp_hom @[elementwise (attr := simp)] theorem binaryCoproductIso_inr_comp_hom (X Y : Type u) : Limits.coprod.inr ≫ (binaryCoproductIso X Y).hom = Sum.inr := colimit.isoColimitCocone_ι_hom (binaryCoproductColimitCocone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_coproduct_iso_inr_comp_hom CategoryTheory.Limits.Types.binaryCoproductIso_inr_comp_hom @[elementwise (attr := simp)] theorem binaryCoproductIso_inl_comp_inv (X Y : Type u) : ↾(Sum.inl : X ⟶ Sum X Y) ≫ (binaryCoproductIso X Y).inv = Limits.coprod.inl := colimit.isoColimitCocone_ι_inv (binaryCoproductColimitCocone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_coproduct_iso_inl_comp_inv CategoryTheory.Limits.Types.binaryCoproductIso_inl_comp_inv @[elementwise (attr := simp)] theorem binaryCoproductIso_inr_comp_inv (X Y : Type u) : ↾(Sum.inr : Y ⟶ Sum X Y) ≫ (binaryCoproductIso X Y).inv = Limits.coprod.inr := colimit.isoColimitCocone_ι_inv (binaryCoproductColimitCocone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_coproduct_iso_inr_comp_inv CategoryTheory.Limits.Types.binaryCoproductIso_inr_comp_inv open Function (Injective) theorem binaryCofan_isColimit_iff {X Y : Type u} (c : BinaryCofan X Y) : Nonempty (IsColimit c) ↔ Injective c.inl ∧ Injective c.inr ∧ IsCompl (Set.range c.inl) (Set.range c.inr) := by classical constructor · rintro ⟨h⟩ rw [← show _ = c.inl from h.comp_coconePointUniqueUpToIso_inv (binaryCoproductColimit X Y) ⟨WalkingPair.left⟩, ← show _ = c.inr from h.comp_coconePointUniqueUpToIso_inv (binaryCoproductColimit X Y) ⟨WalkingPair.right⟩] dsimp [binaryCoproductCocone] refine' ⟨(h.coconePointUniqueUpToIso (binaryCoproductColimit X Y)).symm.toEquiv.injective.comp Sum.inl_injective, (h.coconePointUniqueUpToIso (binaryCoproductColimit X Y)).symm.toEquiv.injective.comp Sum.inr_injective, _⟩ erw [Set.range_comp, ← eq_compl_iff_isCompl, Set.range_comp _ Sum.inr, ← Set.image_compl_eq (h.coconePointUniqueUpToIso (binaryCoproductColimit X Y)).symm.toEquiv.bijective]
simp
theorem binaryCofan_isColimit_iff {X Y : Type u} (c : BinaryCofan X Y) : Nonempty (IsColimit c) ↔ Injective c.inl ∧ Injective c.inr ∧ IsCompl (Set.range c.inl) (Set.range c.inr) := by classical constructor · rintro ⟨h⟩ rw [← show _ = c.inl from h.comp_coconePointUniqueUpToIso_inv (binaryCoproductColimit X Y) ⟨WalkingPair.left⟩, ← show _ = c.inr from h.comp_coconePointUniqueUpToIso_inv (binaryCoproductColimit X Y) ⟨WalkingPair.right⟩] dsimp [binaryCoproductCocone] refine' ⟨(h.coconePointUniqueUpToIso (binaryCoproductColimit X Y)).symm.toEquiv.injective.comp Sum.inl_injective, (h.coconePointUniqueUpToIso (binaryCoproductColimit X Y)).symm.toEquiv.injective.comp Sum.inr_injective, _⟩ erw [Set.range_comp, ← eq_compl_iff_isCompl, Set.range_comp _ Sum.inr, ← Set.image_compl_eq (h.coconePointUniqueUpToIso (binaryCoproductColimit X Y)).symm.toEquiv.bijective]
Mathlib.CategoryTheory.Limits.Shapes.Types.302_0.ctQAUYXLRXnvMGw
theorem binaryCofan_isColimit_iff {X Y : Type u} (c : BinaryCofan X Y) : Nonempty (IsColimit c) ↔ Injective c.inl ∧ Injective c.inr ∧ IsCompl (Set.range c.inl) (Set.range c.inr)
Mathlib_CategoryTheory_Limits_Shapes_Types
case mpr X Y : Type u c : BinaryCofan X Y ⊢ Injective (BinaryCofan.inl c) ∧ Injective (BinaryCofan.inr c) ∧ IsCompl (Set.range (BinaryCofan.inl c)) (Set.range (BinaryCofan.inr c)) → Nonempty (IsColimit c)
/- Copyright (c) 2020 Scott Morrison. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Scott Morrison -/ import Mathlib.CategoryTheory.Limits.Types import Mathlib.CategoryTheory.Limits.Shapes.Products import Mathlib.CategoryTheory.Limits.Shapes.BinaryProducts import Mathlib.CategoryTheory.Limits.Shapes.Terminal import Mathlib.CategoryTheory.ConcreteCategory.Basic import Mathlib.Tactic.CategoryTheory.Elementwise #align_import category_theory.limits.shapes.types from "leanprover-community/mathlib"@"5dc6092d09e5e489106865241986f7f2ad28d4c8" /-! # Special shapes for limits in `Type`. The general shape (co)limits defined in `CategoryTheory.Limits.Types` are intended for use through the limits API, and the actual implementation should mostly be considered "sealed". In this file, we provide definitions of the "standard" special shapes of limits in `Type`, giving the expected definitional implementation: * the terminal object is `PUnit` * the binary product of `X` and `Y` is `X × Y` * the product of a family `f : J → Type` is `Π j, f j` * the coproduct of a family `f : J → Type` is `Σ j, f j` * the binary coproduct of `X` and `Y` is the sum type `X ⊕ Y` * the equalizer of a pair of maps `(g, h)` is the subtype `{x : Y // g x = h x}` * the coequalizer of a pair of maps `(f, g)` is the quotient of `Y` by `∀ x : Y, f x ~ g x` * the pullback of `f : X ⟶ Z` and `g : Y ⟶ Z` is the subtype `{ p : X × Y // f p.1 = g p.2 }` of the product We first construct terms of `IsLimit` and `LimitCone`, and then provide isomorphisms with the types generated by the `HasLimit` API. As an example, when setting up the monoidal category structure on `Type` we use the `Types.terminalLimitCone` and `Types.binaryProductLimitCone` definitions. -/ universe v u open CategoryTheory Limits namespace CategoryTheory.Limits.Types example : HasProducts.{v} (Type v) := inferInstance example [UnivLE.{v, u}] : HasProducts.{v} (Type u) := inferInstance -- This shortcut instance is required in `Mathlib.CategoryTheory.Closed.Types`, -- although I don't understand why, and wish it wasn't. instance : HasProducts.{v} (Type v) := inferInstance /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`. -/ @[simp 1001] theorem pi_lift_π_apply {β : Type v} [Small.{u} β] (f : β → Type u) {P : Type u} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := congr_fun (limit.lift_π (Fan.mk P s) ⟨b⟩) x #align category_theory.limits.types.pi_lift_π_apply CategoryTheory.Limits.Types.pi_lift_π_apply /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`, with specialized universes. -/ theorem pi_lift_π_apply' {β : Type v} (f : β → Type v) {P : Type v} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := by simp #align category_theory.limits.types.pi_lift_π_apply' CategoryTheory.Limits.Types.pi_lift_π_apply' /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`. -/ @[simp 1001] theorem pi_map_π_apply {β : Type v} [Small.{u} β] {f g : β → Type u} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := Limit.map_π_apply.{v, u} _ _ _ #align category_theory.limits.types.pi_map_π_apply CategoryTheory.Limits.Types.pi_map_π_apply /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`, with specialized universes. -/ theorem pi_map_π_apply' {β : Type v} {f g : β → Type v} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := by simp #align category_theory.limits.types.pi_map_π_apply' CategoryTheory.Limits.Types.pi_map_π_apply' /-- The category of types has `PUnit` as a terminal object. -/ def terminalLimitCone : Limits.LimitCone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cone := { pt := PUnit π := (Functor.uniqueFromEmpty _).hom } isLimit := { lift := fun _ _ => PUnit.unit fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext apply Subsingleton.elim } #align category_theory.limits.types.terminal_limit_cone CategoryTheory.Limits.Types.terminalLimitCone /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def terminalIso : ⊤_ Type u ≅ PUnit := limit.isoLimitCone terminalLimitCone.{u, 0} #align category_theory.limits.types.terminal_iso CategoryTheory.Limits.Types.terminalIso /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def isTerminalPunit : IsTerminal (PUnit : Type u) := terminalIsTerminal.ofIso terminalIso #align category_theory.limits.types.is_terminal_punit CategoryTheory.Limits.Types.isTerminalPunit -- porting note: the following three instances have been added to ease -- the automation in a definition in `AlgebraicTopology.SimplicialSet` noncomputable instance : Inhabited (⊤_ (Type u)) := ⟨@terminal.from (Type u) _ _ (ULift (Fin 1)) (ULift.up 0)⟩ instance : Subsingleton (⊤_ (Type u)) := ⟨fun a b => congr_fun (@Subsingleton.elim (_ ⟶ ⊤_ (Type u)) _ (fun _ => a) (fun _ => b)) (ULift.up (0 : Fin 1))⟩ noncomputable instance : Unique (⊤_ (Type u)) := Unique.mk' _ /-- A type is terminal if and only if it contains exactly one element. -/ noncomputable def isTerminalEquivUnique (X : Type u) : IsTerminal X ≃ Unique X := equivOfSubsingletonOfSubsingleton (fun h => ((Iso.toEquiv (terminalIsoIsTerminal h).symm).unique)) (fun _ => IsTerminal.ofIso terminalIsTerminal (Equiv.toIso (Equiv.equivOfUnique _ _))) /-- A type is terminal if and only if it is isomorphic to `PUnit`. -/ noncomputable def isTerminalEquivIsoPUnit (X : Type u) : IsTerminal X ≃ (X ≅ PUnit) := by calc IsTerminal X ≃ Unique X := isTerminalEquivUnique _ _ ≃ (X ≃ PUnit.{u + 1}) := uniqueEquivEquivUnique _ _ _ ≃ (X ≅ PUnit) := equivEquivIso /-- The category of types has `PEmpty` as an initial object. -/ def initialColimitCocone : Limits.ColimitCocone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cocone := { pt := PEmpty ι := (Functor.uniqueFromEmpty _).inv } isColimit := { desc := fun _ => by rintro ⟨⟩ fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext x; cases x } #align category_theory.limits.types.initial_colimit_cocone CategoryTheory.Limits.Types.initialColimitCocone /-- The initial object in `Type u` is `PEmpty`. -/ noncomputable def initialIso : ⊥_ Type u ≅ PEmpty := colimit.isoColimitCocone initialColimitCocone.{u, 0} #align category_theory.limits.types.initial_iso CategoryTheory.Limits.Types.initialIso /-- The initial object in `Type u` is `PEmpty`. -/ noncomputable def isInitialPunit : IsInitial (PEmpty : Type u) := initialIsInitial.ofIso initialIso #align category_theory.limits.types.is_initial_punit CategoryTheory.Limits.Types.isInitialPunit open CategoryTheory.Limits.WalkingPair -- We manually generate the other projection lemmas since the simp-normal form for the legs is -- otherwise not created correctly. /-- The product type `X × Y` forms a cone for the binary product of `X` and `Y`. -/ @[simps! pt] def binaryProductCone (X Y : Type u) : BinaryFan X Y := BinaryFan.mk _root_.Prod.fst _root_.Prod.snd #align category_theory.limits.types.binary_product_cone CategoryTheory.Limits.Types.binaryProductCone @[simp] theorem binaryProductCone_fst (X Y : Type u) : (binaryProductCone X Y).fst = _root_.Prod.fst := rfl #align category_theory.limits.types.binary_product_cone_fst CategoryTheory.Limits.Types.binaryProductCone_fst @[simp] theorem binaryProductCone_snd (X Y : Type u) : (binaryProductCone X Y).snd = _root_.Prod.snd := rfl #align category_theory.limits.types.binary_product_cone_snd CategoryTheory.Limits.Types.binaryProductCone_snd /-- The product type `X × Y` is a binary product for `X` and `Y`. -/ @[simps] def binaryProductLimit (X Y : Type u) : IsLimit (binaryProductCone X Y) where lift (s : BinaryFan X Y) x := (s.fst x, s.snd x) fac _ j := Discrete.recOn j fun j => WalkingPair.casesOn j rfl rfl uniq _ _ w := funext fun x => Prod.ext (congr_fun (w ⟨left⟩) x) (congr_fun (w ⟨right⟩) x) #align category_theory.limits.types.binary_product_limit CategoryTheory.Limits.Types.binaryProductLimit /-- The category of types has `X × Y`, the usual cartesian product, as the binary product of `X` and `Y`. -/ @[simps] def binaryProductLimitCone (X Y : Type u) : Limits.LimitCone (pair X Y) := ⟨_, binaryProductLimit X Y⟩ #align category_theory.limits.types.binary_product_limit_cone CategoryTheory.Limits.Types.binaryProductLimitCone /-- The categorical binary product in `Type u` is cartesian product. -/ noncomputable def binaryProductIso (X Y : Type u) : Limits.prod X Y ≅ X × Y := limit.isoLimitCone (binaryProductLimitCone X Y) #align category_theory.limits.types.binary_product_iso CategoryTheory.Limits.Types.binaryProductIso @[elementwise (attr := simp)] theorem binaryProductIso_hom_comp_fst (X Y : Type u) : (binaryProductIso X Y).hom ≫ _root_.Prod.fst = Limits.prod.fst := limit.isoLimitCone_hom_π (binaryProductLimitCone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_product_iso_hom_comp_fst CategoryTheory.Limits.Types.binaryProductIso_hom_comp_fst @[elementwise (attr := simp)] theorem binaryProductIso_hom_comp_snd (X Y : Type u) : (binaryProductIso X Y).hom ≫ _root_.Prod.snd = Limits.prod.snd := limit.isoLimitCone_hom_π (binaryProductLimitCone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_product_iso_hom_comp_snd CategoryTheory.Limits.Types.binaryProductIso_hom_comp_snd @[elementwise (attr := simp)] theorem binaryProductIso_inv_comp_fst (X Y : Type u) : (binaryProductIso X Y).inv ≫ Limits.prod.fst = _root_.Prod.fst := limit.isoLimitCone_inv_π (binaryProductLimitCone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_product_iso_inv_comp_fst CategoryTheory.Limits.Types.binaryProductIso_inv_comp_fst @[elementwise (attr := simp)] theorem binaryProductIso_inv_comp_snd (X Y : Type u) : (binaryProductIso X Y).inv ≫ Limits.prod.snd = _root_.Prod.snd := limit.isoLimitCone_inv_π (binaryProductLimitCone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_product_iso_inv_comp_snd CategoryTheory.Limits.Types.binaryProductIso_inv_comp_snd -- porting note: it was originally @[simps (config := { typeMd := reducible })] -- We add the option `type_md` to tell `@[simps]` to not treat homomorphisms `X ⟶ Y` in `Type*` as -- a function type /-- The functor which sends `X, Y` to the product type `X × Y`. -/ @[simps] def binaryProductFunctor : Type u ⥤ Type u ⥤ Type u where obj X := { obj := fun Y => X × Y map := fun { Y₁ Y₂} f => (binaryProductLimit X Y₂).lift (BinaryFan.mk _root_.Prod.fst (_root_.Prod.snd ≫ f)) } map {X₁ X₂} f := { app := fun Y => (binaryProductLimit X₂ Y).lift (BinaryFan.mk (_root_.Prod.fst ≫ f) _root_.Prod.snd) } #align category_theory.limits.types.binary_product_functor CategoryTheory.Limits.Types.binaryProductFunctor /-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _) := by refine' NatIso.ofComponents (fun X => _) (fun _ => _) · refine' NatIso.ofComponents (fun Y => _) (fun _ => _) · exact ((limit.isLimit _).conePointUniqueUpToIso (binaryProductLimit X Y)).symm · apply Limits.prod.hom_ext <;> simp <;> rfl · ext : 2 apply Limits.prod.hom_ext <;> simp <;> rfl #align category_theory.limits.types.binary_product_iso_prod CategoryTheory.Limits.Types.binaryProductIsoProd /-- The sum type `X ⊕ Y` forms a cocone for the binary coproduct of `X` and `Y`. -/ @[simps!] def binaryCoproductCocone (X Y : Type u) : Cocone (pair X Y) := BinaryCofan.mk Sum.inl Sum.inr #align category_theory.limits.types.binary_coproduct_cocone CategoryTheory.Limits.Types.binaryCoproductCocone /-- The sum type `X ⊕ Y` is a binary coproduct for `X` and `Y`. -/ @[simps] def binaryCoproductColimit (X Y : Type u) : IsColimit (binaryCoproductCocone X Y) where desc := fun s : BinaryCofan X Y => Sum.elim s.inl s.inr fac _ j := Discrete.recOn j fun j => WalkingPair.casesOn j rfl rfl uniq _ _ w := funext fun x => Sum.casesOn x (congr_fun (w ⟨left⟩)) (congr_fun (w ⟨right⟩)) #align category_theory.limits.types.binary_coproduct_colimit CategoryTheory.Limits.Types.binaryCoproductColimit /-- The category of types has `X ⊕ Y`, as the binary coproduct of `X` and `Y`. -/ def binaryCoproductColimitCocone (X Y : Type u) : Limits.ColimitCocone (pair X Y) := ⟨_, binaryCoproductColimit X Y⟩ #align category_theory.limits.types.binary_coproduct_colimit_cocone CategoryTheory.Limits.Types.binaryCoproductColimitCocone /-- The categorical binary coproduct in `Type u` is the sum `X ⊕ Y`. -/ noncomputable def binaryCoproductIso (X Y : Type u) : Limits.coprod X Y ≅ Sum X Y := colimit.isoColimitCocone (binaryCoproductColimitCocone X Y) #align category_theory.limits.types.binary_coproduct_iso CategoryTheory.Limits.Types.binaryCoproductIso --open CategoryTheory.Type @[elementwise (attr := simp)] theorem binaryCoproductIso_inl_comp_hom (X Y : Type u) : Limits.coprod.inl ≫ (binaryCoproductIso X Y).hom = Sum.inl := colimit.isoColimitCocone_ι_hom (binaryCoproductColimitCocone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_coproduct_iso_inl_comp_hom CategoryTheory.Limits.Types.binaryCoproductIso_inl_comp_hom @[elementwise (attr := simp)] theorem binaryCoproductIso_inr_comp_hom (X Y : Type u) : Limits.coprod.inr ≫ (binaryCoproductIso X Y).hom = Sum.inr := colimit.isoColimitCocone_ι_hom (binaryCoproductColimitCocone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_coproduct_iso_inr_comp_hom CategoryTheory.Limits.Types.binaryCoproductIso_inr_comp_hom @[elementwise (attr := simp)] theorem binaryCoproductIso_inl_comp_inv (X Y : Type u) : ↾(Sum.inl : X ⟶ Sum X Y) ≫ (binaryCoproductIso X Y).inv = Limits.coprod.inl := colimit.isoColimitCocone_ι_inv (binaryCoproductColimitCocone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_coproduct_iso_inl_comp_inv CategoryTheory.Limits.Types.binaryCoproductIso_inl_comp_inv @[elementwise (attr := simp)] theorem binaryCoproductIso_inr_comp_inv (X Y : Type u) : ↾(Sum.inr : Y ⟶ Sum X Y) ≫ (binaryCoproductIso X Y).inv = Limits.coprod.inr := colimit.isoColimitCocone_ι_inv (binaryCoproductColimitCocone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_coproduct_iso_inr_comp_inv CategoryTheory.Limits.Types.binaryCoproductIso_inr_comp_inv open Function (Injective) theorem binaryCofan_isColimit_iff {X Y : Type u} (c : BinaryCofan X Y) : Nonempty (IsColimit c) ↔ Injective c.inl ∧ Injective c.inr ∧ IsCompl (Set.range c.inl) (Set.range c.inr) := by classical constructor · rintro ⟨h⟩ rw [← show _ = c.inl from h.comp_coconePointUniqueUpToIso_inv (binaryCoproductColimit X Y) ⟨WalkingPair.left⟩, ← show _ = c.inr from h.comp_coconePointUniqueUpToIso_inv (binaryCoproductColimit X Y) ⟨WalkingPair.right⟩] dsimp [binaryCoproductCocone] refine' ⟨(h.coconePointUniqueUpToIso (binaryCoproductColimit X Y)).symm.toEquiv.injective.comp Sum.inl_injective, (h.coconePointUniqueUpToIso (binaryCoproductColimit X Y)).symm.toEquiv.injective.comp Sum.inr_injective, _⟩ erw [Set.range_comp, ← eq_compl_iff_isCompl, Set.range_comp _ Sum.inr, ← Set.image_compl_eq (h.coconePointUniqueUpToIso (binaryCoproductColimit X Y)).symm.toEquiv.bijective] simp ·
rintro ⟨h₁, h₂, h₃⟩
theorem binaryCofan_isColimit_iff {X Y : Type u} (c : BinaryCofan X Y) : Nonempty (IsColimit c) ↔ Injective c.inl ∧ Injective c.inr ∧ IsCompl (Set.range c.inl) (Set.range c.inr) := by classical constructor · rintro ⟨h⟩ rw [← show _ = c.inl from h.comp_coconePointUniqueUpToIso_inv (binaryCoproductColimit X Y) ⟨WalkingPair.left⟩, ← show _ = c.inr from h.comp_coconePointUniqueUpToIso_inv (binaryCoproductColimit X Y) ⟨WalkingPair.right⟩] dsimp [binaryCoproductCocone] refine' ⟨(h.coconePointUniqueUpToIso (binaryCoproductColimit X Y)).symm.toEquiv.injective.comp Sum.inl_injective, (h.coconePointUniqueUpToIso (binaryCoproductColimit X Y)).symm.toEquiv.injective.comp Sum.inr_injective, _⟩ erw [Set.range_comp, ← eq_compl_iff_isCompl, Set.range_comp _ Sum.inr, ← Set.image_compl_eq (h.coconePointUniqueUpToIso (binaryCoproductColimit X Y)).symm.toEquiv.bijective] simp ·
Mathlib.CategoryTheory.Limits.Shapes.Types.302_0.ctQAUYXLRXnvMGw
theorem binaryCofan_isColimit_iff {X Y : Type u} (c : BinaryCofan X Y) : Nonempty (IsColimit c) ↔ Injective c.inl ∧ Injective c.inr ∧ IsCompl (Set.range c.inl) (Set.range c.inr)
Mathlib_CategoryTheory_Limits_Shapes_Types
case mpr.intro.intro X Y : Type u c : BinaryCofan X Y h₁ : Injective (BinaryCofan.inl c) h₂ : Injective (BinaryCofan.inr c) h₃ : IsCompl (Set.range (BinaryCofan.inl c)) (Set.range (BinaryCofan.inr c)) ⊢ Nonempty (IsColimit c)
/- Copyright (c) 2020 Scott Morrison. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Scott Morrison -/ import Mathlib.CategoryTheory.Limits.Types import Mathlib.CategoryTheory.Limits.Shapes.Products import Mathlib.CategoryTheory.Limits.Shapes.BinaryProducts import Mathlib.CategoryTheory.Limits.Shapes.Terminal import Mathlib.CategoryTheory.ConcreteCategory.Basic import Mathlib.Tactic.CategoryTheory.Elementwise #align_import category_theory.limits.shapes.types from "leanprover-community/mathlib"@"5dc6092d09e5e489106865241986f7f2ad28d4c8" /-! # Special shapes for limits in `Type`. The general shape (co)limits defined in `CategoryTheory.Limits.Types` are intended for use through the limits API, and the actual implementation should mostly be considered "sealed". In this file, we provide definitions of the "standard" special shapes of limits in `Type`, giving the expected definitional implementation: * the terminal object is `PUnit` * the binary product of `X` and `Y` is `X × Y` * the product of a family `f : J → Type` is `Π j, f j` * the coproduct of a family `f : J → Type` is `Σ j, f j` * the binary coproduct of `X` and `Y` is the sum type `X ⊕ Y` * the equalizer of a pair of maps `(g, h)` is the subtype `{x : Y // g x = h x}` * the coequalizer of a pair of maps `(f, g)` is the quotient of `Y` by `∀ x : Y, f x ~ g x` * the pullback of `f : X ⟶ Z` and `g : Y ⟶ Z` is the subtype `{ p : X × Y // f p.1 = g p.2 }` of the product We first construct terms of `IsLimit` and `LimitCone`, and then provide isomorphisms with the types generated by the `HasLimit` API. As an example, when setting up the monoidal category structure on `Type` we use the `Types.terminalLimitCone` and `Types.binaryProductLimitCone` definitions. -/ universe v u open CategoryTheory Limits namespace CategoryTheory.Limits.Types example : HasProducts.{v} (Type v) := inferInstance example [UnivLE.{v, u}] : HasProducts.{v} (Type u) := inferInstance -- This shortcut instance is required in `Mathlib.CategoryTheory.Closed.Types`, -- although I don't understand why, and wish it wasn't. instance : HasProducts.{v} (Type v) := inferInstance /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`. -/ @[simp 1001] theorem pi_lift_π_apply {β : Type v} [Small.{u} β] (f : β → Type u) {P : Type u} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := congr_fun (limit.lift_π (Fan.mk P s) ⟨b⟩) x #align category_theory.limits.types.pi_lift_π_apply CategoryTheory.Limits.Types.pi_lift_π_apply /-- A restatement of `Types.Limit.lift_π_apply` that uses `Pi.π` and `Pi.lift`, with specialized universes. -/ theorem pi_lift_π_apply' {β : Type v} (f : β → Type v) {P : Type v} (s : ∀ b, P ⟶ f b) (b : β) (x : P) : (Pi.π f b : (piObj f) → f b) (@Pi.lift β _ _ f _ P s x) = s b x := by simp #align category_theory.limits.types.pi_lift_π_apply' CategoryTheory.Limits.Types.pi_lift_π_apply' /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`. -/ @[simp 1001] theorem pi_map_π_apply {β : Type v} [Small.{u} β] {f g : β → Type u} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := Limit.map_π_apply.{v, u} _ _ _ #align category_theory.limits.types.pi_map_π_apply CategoryTheory.Limits.Types.pi_map_π_apply /-- A restatement of `Types.Limit.map_π_apply` that uses `Pi.π` and `Pi.map`, with specialized universes. -/ theorem pi_map_π_apply' {β : Type v} {f g : β → Type v} (α : ∀ j, f j ⟶ g j) (b : β) (x) : (Pi.π g b : ∏ g → g b) (Pi.map α x) = α b ((Pi.π f b : ∏ f → f b) x) := by simp #align category_theory.limits.types.pi_map_π_apply' CategoryTheory.Limits.Types.pi_map_π_apply' /-- The category of types has `PUnit` as a terminal object. -/ def terminalLimitCone : Limits.LimitCone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cone := { pt := PUnit π := (Functor.uniqueFromEmpty _).hom } isLimit := { lift := fun _ _ => PUnit.unit fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext apply Subsingleton.elim } #align category_theory.limits.types.terminal_limit_cone CategoryTheory.Limits.Types.terminalLimitCone /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def terminalIso : ⊤_ Type u ≅ PUnit := limit.isoLimitCone terminalLimitCone.{u, 0} #align category_theory.limits.types.terminal_iso CategoryTheory.Limits.Types.terminalIso /-- The terminal object in `Type u` is `PUnit`. -/ noncomputable def isTerminalPunit : IsTerminal (PUnit : Type u) := terminalIsTerminal.ofIso terminalIso #align category_theory.limits.types.is_terminal_punit CategoryTheory.Limits.Types.isTerminalPunit -- porting note: the following three instances have been added to ease -- the automation in a definition in `AlgebraicTopology.SimplicialSet` noncomputable instance : Inhabited (⊤_ (Type u)) := ⟨@terminal.from (Type u) _ _ (ULift (Fin 1)) (ULift.up 0)⟩ instance : Subsingleton (⊤_ (Type u)) := ⟨fun a b => congr_fun (@Subsingleton.elim (_ ⟶ ⊤_ (Type u)) _ (fun _ => a) (fun _ => b)) (ULift.up (0 : Fin 1))⟩ noncomputable instance : Unique (⊤_ (Type u)) := Unique.mk' _ /-- A type is terminal if and only if it contains exactly one element. -/ noncomputable def isTerminalEquivUnique (X : Type u) : IsTerminal X ≃ Unique X := equivOfSubsingletonOfSubsingleton (fun h => ((Iso.toEquiv (terminalIsoIsTerminal h).symm).unique)) (fun _ => IsTerminal.ofIso terminalIsTerminal (Equiv.toIso (Equiv.equivOfUnique _ _))) /-- A type is terminal if and only if it is isomorphic to `PUnit`. -/ noncomputable def isTerminalEquivIsoPUnit (X : Type u) : IsTerminal X ≃ (X ≅ PUnit) := by calc IsTerminal X ≃ Unique X := isTerminalEquivUnique _ _ ≃ (X ≃ PUnit.{u + 1}) := uniqueEquivEquivUnique _ _ _ ≃ (X ≅ PUnit) := equivEquivIso /-- The category of types has `PEmpty` as an initial object. -/ def initialColimitCocone : Limits.ColimitCocone (Functor.empty (Type u)) where -- porting note: tidy was able to fill the structure automatically cocone := { pt := PEmpty ι := (Functor.uniqueFromEmpty _).inv } isColimit := { desc := fun _ => by rintro ⟨⟩ fac := fun _ => by rintro ⟨⟨⟩⟩ uniq := fun _ _ _ => by funext x; cases x } #align category_theory.limits.types.initial_colimit_cocone CategoryTheory.Limits.Types.initialColimitCocone /-- The initial object in `Type u` is `PEmpty`. -/ noncomputable def initialIso : ⊥_ Type u ≅ PEmpty := colimit.isoColimitCocone initialColimitCocone.{u, 0} #align category_theory.limits.types.initial_iso CategoryTheory.Limits.Types.initialIso /-- The initial object in `Type u` is `PEmpty`. -/ noncomputable def isInitialPunit : IsInitial (PEmpty : Type u) := initialIsInitial.ofIso initialIso #align category_theory.limits.types.is_initial_punit CategoryTheory.Limits.Types.isInitialPunit open CategoryTheory.Limits.WalkingPair -- We manually generate the other projection lemmas since the simp-normal form for the legs is -- otherwise not created correctly. /-- The product type `X × Y` forms a cone for the binary product of `X` and `Y`. -/ @[simps! pt] def binaryProductCone (X Y : Type u) : BinaryFan X Y := BinaryFan.mk _root_.Prod.fst _root_.Prod.snd #align category_theory.limits.types.binary_product_cone CategoryTheory.Limits.Types.binaryProductCone @[simp] theorem binaryProductCone_fst (X Y : Type u) : (binaryProductCone X Y).fst = _root_.Prod.fst := rfl #align category_theory.limits.types.binary_product_cone_fst CategoryTheory.Limits.Types.binaryProductCone_fst @[simp] theorem binaryProductCone_snd (X Y : Type u) : (binaryProductCone X Y).snd = _root_.Prod.snd := rfl #align category_theory.limits.types.binary_product_cone_snd CategoryTheory.Limits.Types.binaryProductCone_snd /-- The product type `X × Y` is a binary product for `X` and `Y`. -/ @[simps] def binaryProductLimit (X Y : Type u) : IsLimit (binaryProductCone X Y) where lift (s : BinaryFan X Y) x := (s.fst x, s.snd x) fac _ j := Discrete.recOn j fun j => WalkingPair.casesOn j rfl rfl uniq _ _ w := funext fun x => Prod.ext (congr_fun (w ⟨left⟩) x) (congr_fun (w ⟨right⟩) x) #align category_theory.limits.types.binary_product_limit CategoryTheory.Limits.Types.binaryProductLimit /-- The category of types has `X × Y`, the usual cartesian product, as the binary product of `X` and `Y`. -/ @[simps] def binaryProductLimitCone (X Y : Type u) : Limits.LimitCone (pair X Y) := ⟨_, binaryProductLimit X Y⟩ #align category_theory.limits.types.binary_product_limit_cone CategoryTheory.Limits.Types.binaryProductLimitCone /-- The categorical binary product in `Type u` is cartesian product. -/ noncomputable def binaryProductIso (X Y : Type u) : Limits.prod X Y ≅ X × Y := limit.isoLimitCone (binaryProductLimitCone X Y) #align category_theory.limits.types.binary_product_iso CategoryTheory.Limits.Types.binaryProductIso @[elementwise (attr := simp)] theorem binaryProductIso_hom_comp_fst (X Y : Type u) : (binaryProductIso X Y).hom ≫ _root_.Prod.fst = Limits.prod.fst := limit.isoLimitCone_hom_π (binaryProductLimitCone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_product_iso_hom_comp_fst CategoryTheory.Limits.Types.binaryProductIso_hom_comp_fst @[elementwise (attr := simp)] theorem binaryProductIso_hom_comp_snd (X Y : Type u) : (binaryProductIso X Y).hom ≫ _root_.Prod.snd = Limits.prod.snd := limit.isoLimitCone_hom_π (binaryProductLimitCone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_product_iso_hom_comp_snd CategoryTheory.Limits.Types.binaryProductIso_hom_comp_snd @[elementwise (attr := simp)] theorem binaryProductIso_inv_comp_fst (X Y : Type u) : (binaryProductIso X Y).inv ≫ Limits.prod.fst = _root_.Prod.fst := limit.isoLimitCone_inv_π (binaryProductLimitCone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_product_iso_inv_comp_fst CategoryTheory.Limits.Types.binaryProductIso_inv_comp_fst @[elementwise (attr := simp)] theorem binaryProductIso_inv_comp_snd (X Y : Type u) : (binaryProductIso X Y).inv ≫ Limits.prod.snd = _root_.Prod.snd := limit.isoLimitCone_inv_π (binaryProductLimitCone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_product_iso_inv_comp_snd CategoryTheory.Limits.Types.binaryProductIso_inv_comp_snd -- porting note: it was originally @[simps (config := { typeMd := reducible })] -- We add the option `type_md` to tell `@[simps]` to not treat homomorphisms `X ⟶ Y` in `Type*` as -- a function type /-- The functor which sends `X, Y` to the product type `X × Y`. -/ @[simps] def binaryProductFunctor : Type u ⥤ Type u ⥤ Type u where obj X := { obj := fun Y => X × Y map := fun { Y₁ Y₂} f => (binaryProductLimit X Y₂).lift (BinaryFan.mk _root_.Prod.fst (_root_.Prod.snd ≫ f)) } map {X₁ X₂} f := { app := fun Y => (binaryProductLimit X₂ Y).lift (BinaryFan.mk (_root_.Prod.fst ≫ f) _root_.Prod.snd) } #align category_theory.limits.types.binary_product_functor CategoryTheory.Limits.Types.binaryProductFunctor /-- The product functor given by the instance `HasBinaryProducts (Type u)` is isomorphic to the explicit binary product functor given by the product type. -/ noncomputable def binaryProductIsoProd : binaryProductFunctor ≅ (prod.functor : Type u ⥤ _) := by refine' NatIso.ofComponents (fun X => _) (fun _ => _) · refine' NatIso.ofComponents (fun Y => _) (fun _ => _) · exact ((limit.isLimit _).conePointUniqueUpToIso (binaryProductLimit X Y)).symm · apply Limits.prod.hom_ext <;> simp <;> rfl · ext : 2 apply Limits.prod.hom_ext <;> simp <;> rfl #align category_theory.limits.types.binary_product_iso_prod CategoryTheory.Limits.Types.binaryProductIsoProd /-- The sum type `X ⊕ Y` forms a cocone for the binary coproduct of `X` and `Y`. -/ @[simps!] def binaryCoproductCocone (X Y : Type u) : Cocone (pair X Y) := BinaryCofan.mk Sum.inl Sum.inr #align category_theory.limits.types.binary_coproduct_cocone CategoryTheory.Limits.Types.binaryCoproductCocone /-- The sum type `X ⊕ Y` is a binary coproduct for `X` and `Y`. -/ @[simps] def binaryCoproductColimit (X Y : Type u) : IsColimit (binaryCoproductCocone X Y) where desc := fun s : BinaryCofan X Y => Sum.elim s.inl s.inr fac _ j := Discrete.recOn j fun j => WalkingPair.casesOn j rfl rfl uniq _ _ w := funext fun x => Sum.casesOn x (congr_fun (w ⟨left⟩)) (congr_fun (w ⟨right⟩)) #align category_theory.limits.types.binary_coproduct_colimit CategoryTheory.Limits.Types.binaryCoproductColimit /-- The category of types has `X ⊕ Y`, as the binary coproduct of `X` and `Y`. -/ def binaryCoproductColimitCocone (X Y : Type u) : Limits.ColimitCocone (pair X Y) := ⟨_, binaryCoproductColimit X Y⟩ #align category_theory.limits.types.binary_coproduct_colimit_cocone CategoryTheory.Limits.Types.binaryCoproductColimitCocone /-- The categorical binary coproduct in `Type u` is the sum `X ⊕ Y`. -/ noncomputable def binaryCoproductIso (X Y : Type u) : Limits.coprod X Y ≅ Sum X Y := colimit.isoColimitCocone (binaryCoproductColimitCocone X Y) #align category_theory.limits.types.binary_coproduct_iso CategoryTheory.Limits.Types.binaryCoproductIso --open CategoryTheory.Type @[elementwise (attr := simp)] theorem binaryCoproductIso_inl_comp_hom (X Y : Type u) : Limits.coprod.inl ≫ (binaryCoproductIso X Y).hom = Sum.inl := colimit.isoColimitCocone_ι_hom (binaryCoproductColimitCocone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_coproduct_iso_inl_comp_hom CategoryTheory.Limits.Types.binaryCoproductIso_inl_comp_hom @[elementwise (attr := simp)] theorem binaryCoproductIso_inr_comp_hom (X Y : Type u) : Limits.coprod.inr ≫ (binaryCoproductIso X Y).hom = Sum.inr := colimit.isoColimitCocone_ι_hom (binaryCoproductColimitCocone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_coproduct_iso_inr_comp_hom CategoryTheory.Limits.Types.binaryCoproductIso_inr_comp_hom @[elementwise (attr := simp)] theorem binaryCoproductIso_inl_comp_inv (X Y : Type u) : ↾(Sum.inl : X ⟶ Sum X Y) ≫ (binaryCoproductIso X Y).inv = Limits.coprod.inl := colimit.isoColimitCocone_ι_inv (binaryCoproductColimitCocone X Y) ⟨WalkingPair.left⟩ #align category_theory.limits.types.binary_coproduct_iso_inl_comp_inv CategoryTheory.Limits.Types.binaryCoproductIso_inl_comp_inv @[elementwise (attr := simp)] theorem binaryCoproductIso_inr_comp_inv (X Y : Type u) : ↾(Sum.inr : Y ⟶ Sum X Y) ≫ (binaryCoproductIso X Y).inv = Limits.coprod.inr := colimit.isoColimitCocone_ι_inv (binaryCoproductColimitCocone X Y) ⟨WalkingPair.right⟩ #align category_theory.limits.types.binary_coproduct_iso_inr_comp_inv CategoryTheory.Limits.Types.binaryCoproductIso_inr_comp_inv open Function (Injective) theorem binaryCofan_isColimit_iff {X Y : Type u} (c : BinaryCofan X Y) : Nonempty (IsColimit c) ↔ Injective c.inl ∧ Injective c.inr ∧ IsCompl (Set.range c.inl) (Set.range c.inr) := by classical constructor · rintro ⟨h⟩ rw [← show _ = c.inl from h.comp_coconePointUniqueUpToIso_inv (binaryCoproductColimit X Y) ⟨WalkingPair.left⟩, ← show _ = c.inr from h.comp_coconePointUniqueUpToIso_inv (binaryCoproductColimit X Y) ⟨WalkingPair.right⟩] dsimp [binaryCoproductCocone] refine' ⟨(h.coconePointUniqueUpToIso (binaryCoproductColimit X Y)).symm.toEquiv.injective.comp Sum.inl_injective, (h.coconePointUniqueUpToIso (binaryCoproductColimit X Y)).symm.toEquiv.injective.comp Sum.inr_injective, _⟩ erw [Set.range_comp, ← eq_compl_iff_isCompl, Set.range_comp _ Sum.inr, ← Set.image_compl_eq (h.coconePointUniqueUpToIso (binaryCoproductColimit X Y)).symm.toEquiv.bijective] simp · rintro ⟨h₁, h₂, h₃⟩
have : ∀ x, x ∈ Set.range c.inl ∨ x ∈ Set.range c.inr := by rw [eq_compl_iff_isCompl.mpr h₃.symm] exact fun _ => or_not
theorem binaryCofan_isColimit_iff {X Y : Type u} (c : BinaryCofan X Y) : Nonempty (IsColimit c) ↔ Injective c.inl ∧ Injective c.inr ∧ IsCompl (Set.range c.inl) (Set.range c.inr) := by classical constructor · rintro ⟨h⟩ rw [← show _ = c.inl from h.comp_coconePointUniqueUpToIso_inv (binaryCoproductColimit X Y) ⟨WalkingPair.left⟩, ← show _ = c.inr from h.comp_coconePointUniqueUpToIso_inv (binaryCoproductColimit X Y) ⟨WalkingPair.right⟩] dsimp [binaryCoproductCocone] refine' ⟨(h.coconePointUniqueUpToIso (binaryCoproductColimit X Y)).symm.toEquiv.injective.comp Sum.inl_injective, (h.coconePointUniqueUpToIso (binaryCoproductColimit X Y)).symm.toEquiv.injective.comp Sum.inr_injective, _⟩ erw [Set.range_comp, ← eq_compl_iff_isCompl, Set.range_comp _ Sum.inr, ← Set.image_compl_eq (h.coconePointUniqueUpToIso (binaryCoproductColimit X Y)).symm.toEquiv.bijective] simp · rintro ⟨h₁, h₂, h₃⟩
Mathlib.CategoryTheory.Limits.Shapes.Types.302_0.ctQAUYXLRXnvMGw
theorem binaryCofan_isColimit_iff {X Y : Type u} (c : BinaryCofan X Y) : Nonempty (IsColimit c) ↔ Injective c.inl ∧ Injective c.inr ∧ IsCompl (Set.range c.inl) (Set.range c.inr)
Mathlib_CategoryTheory_Limits_Shapes_Types