Skip to content

Commit

Permalink
fix merge
Browse files Browse the repository at this point in the history
  • Loading branch information
vihdzp committed Sep 17, 2024
1 parent e9076ac commit e7bb46a
Showing 1 changed file with 2 additions and 1 deletion.
3 changes: 2 additions & 1 deletion Mathlib/SetTheory/Game/Nim.lean
Original file line number Diff line number Diff line change
Expand Up @@ -226,7 +226,8 @@ theorem grundyValue_eq_mex_left (G : PGame) :
theorem grundyValue_ne_moveLeft {G : PGame} (i : G.LeftMoves) :
grundyValue (G.moveLeft i) ≠ grundyValue G := by
conv_rhs => rw [grundyValue_eq_sInf_moveLeft]
have := csInf_mem (compl_nonempty_of_small (Set.range fun i => grundyValue (G.moveLeft i)))
have := csInf_mem (nonempty_of_not_bddAbove <|
not_bddAbove_compl_of_small (Set.range fun i => grundyValue (G.moveLeft i)))
rw [Set.mem_compl_iff, Set.mem_range, not_exists] at this
exact this _

Expand Down

0 comments on commit e7bb46a

Please sign in to comment.