Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit 0bea7a0

Browse files
committed
feat(set_theory/pgame): Lemmas about order and left/right moves (#13590)
1 parent 26b2d72 commit 0bea7a0

File tree

1 file changed

+16
-0
lines changed

1 file changed

+16
-0
lines changed

src/set_theory/game/pgame.lean

Lines changed: 16 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -352,6 +352,22 @@ theorem lt_mk_of_le {x : pgame} {yl yr : Type*} {yL : yl → pgame} {yR i} :
352352
(x ≤ yL i) → x < ⟨yl, yr, yL, yR⟩ :=
353353
by { cases x, rw mk_lt_mk, exact λ h, or.inl ⟨_, h⟩ }
354354

355+
theorem move_left_lt_of_le {x y : pgame} {i} :
356+
x ≤ y → x.move_left i < y :=
357+
by { cases x, exact lt_of_le_mk }
358+
359+
theorem lt_move_right_of_le {x y : pgame} {i} :
360+
x ≤ y → x < y.move_right i :=
361+
by { cases y, exact lt_of_mk_le }
362+
363+
theorem lt_of_move_right_le {x y : pgame} {i} :
364+
x.move_right i ≤ y → x < y :=
365+
by { cases x, rw move_right_mk, exact mk_lt_of_le }
366+
367+
theorem lt_of_le_move_left {x y : pgame} {i} :
368+
x ≤ y.move_left i → x < y :=
369+
by { cases y, rw move_left_mk, exact lt_mk_of_le }
370+
355371
private theorem not_le_lt {x y : pgame} :
356372
(¬ x ≤ y ↔ y < x) ∧ (¬ x < y ↔ y ≤ x) :=
357373
begin

0 commit comments

Comments
 (0)