Skip to content

Commit

Permalink
feat(set_theory/game/impartial): Relabelling of impartial game is imp…
Browse files Browse the repository at this point in the history
…artial (#13843)
  • Loading branch information
vihdzp committed May 1, 2022
1 parent 4b92515 commit 51b1e11
Showing 1 changed file with 13 additions and 0 deletions.
13 changes: 13 additions & 0 deletions src/set_theory/game/impartial.lean
Expand Up @@ -56,6 +56,19 @@ instance move_right_impartial {G : pgame} [h : G.impartial] (j : G.right_moves)
(G.move_right j).impartial :=
(impartial_def.1 h).2.2 j

theorem impartial_congr : ∀ {G H : pgame} (e : relabelling G H) [G.impartial], H.impartial
| G H e := begin
introI h,
rw impartial_def,
refine ⟨equiv_trans e.symm.equiv (equiv_trans (neg_equiv_self G) (neg_congr e.equiv)),
λ i, _, λ j, _⟩;
cases e with _ _ L R hL hR,
{ convert impartial_congr (hL (L.symm i)),
rw equiv.apply_symm_apply },
{ exact impartial_congr (hR j) }
end
using_well_founded { dec_tac := pgame_wf_tac }

instance impartial_add : ∀ (G H : pgame) [G.impartial] [H.impartial], (G + H).impartial
| G H :=
begin
Expand Down

0 comments on commit 51b1e11

Please sign in to comment.