Skip to content

Commit

Permalink
feat(set_theory/game/pgame): simp + private (#13596)
Browse files Browse the repository at this point in the history
  • Loading branch information
vihdzp committed Apr 22, 2022
1 parent 62205c2 commit 6729cca
Showing 1 changed file with 3 additions and 3 deletions.
6 changes: 3 additions & 3 deletions src/set_theory/game/pgame.lean
Expand Up @@ -347,7 +347,7 @@ 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 not_le_lt {x y : pgame} :
private theorem not_le_lt {x y : pgame} :
(¬ x ≤ y ↔ y < x) ∧ (¬ x < y ↔ y ≤ x) :=
begin
induction x with xl xr xL xR IHxl IHxr generalizing y,
Expand All @@ -358,8 +358,8 @@ begin
and_comm, or_comm, IHxl, IHxr, IHyl, IHyr, iff_self, and_self]
end

theorem not_le {x y : pgame} : ¬ x ≤ y ↔ y < x := not_le_lt.1
theorem not_lt {x y : pgame} : ¬ x < y ↔ y ≤ x := not_le_lt.2
@[simp] theorem not_le {x y : pgame} : ¬ x ≤ y ↔ y < x := not_le_lt.1
@[simp] theorem not_lt {x y : pgame} : ¬ x < y ↔ y ≤ x := not_le_lt.2

@[refl] protected theorem le_refl : ∀ x : pgame, x ≤ x
| ⟨l, r, L, R⟩ := by rw mk_le_mk; exact
Expand Down

0 comments on commit 6729cca

Please sign in to comment.