Skip to content

Commit

Permalink
feat(set_theory/pgame): Lemmas about order and left/right moves (#13590)
Browse files Browse the repository at this point in the history
  • Loading branch information
vihdzp committed Apr 23, 2022
1 parent 26b2d72 commit 0bea7a0
Showing 1 changed file with 16 additions and 0 deletions.
16 changes: 16 additions & 0 deletions src/set_theory/game/pgame.lean
Original file line number Diff line number Diff line change
Expand Up @@ -352,6 +352,22 @@ theorem lt_mk_of_le {x : pgame} {yl yr : Type*} {yL : yl → pgame} {yR i} :
(x ≤ yL i) → x < ⟨yl, yr, yL, yR⟩ :=
by { cases x, rw mk_lt_mk, exact λ h, or.inl ⟨_, h⟩ }

theorem move_left_lt_of_le {x y : pgame} {i} :
x ≤ y → x.move_left i < y :=
by { cases x, exact lt_of_le_mk }

theorem lt_move_right_of_le {x y : pgame} {i} :
x ≤ y → x < y.move_right i :=
by { cases y, exact lt_of_mk_le }

theorem lt_of_move_right_le {x y : pgame} {i} :
x.move_right i ≤ y → x < y :=
by { cases x, rw move_right_mk, exact mk_lt_of_le }

theorem lt_of_le_move_left {x y : pgame} {i} :
x ≤ y.move_left i → x < y :=
by { cases y, rw move_left_mk, exact lt_mk_of_le }

private theorem not_le_lt {x y : pgame} :
(¬ x ≤ y ↔ y < x) ∧ (¬ x < y ↔ y ≤ x) :=
begin
Expand Down

0 comments on commit 0bea7a0

Please sign in to comment.