Skip to content

Commit

Permalink
feat(set_theory/surreal/basic): add pgame.numeric.left_lt_right (#1…
Browse files Browse the repository at this point in the history
…3809)

Also compress some trivial proofs into a single line
  • Loading branch information
vihdzp committed Apr 29, 2022
1 parent a70166a commit 24bc2e1
Showing 1 changed file with 5 additions and 8 deletions.
13 changes: 5 additions & 8 deletions src/set_theory/surreal/basic.lean
Expand Up @@ -56,18 +56,15 @@ lemma numeric_def (x : pgame) : numeric x ↔ (∀ i j, x.move_left i < x.move_r
(∀ i, numeric (x.move_left i)) ∧ (∀ i, numeric (x.move_right i)) :=
by { cases x, refl }

lemma numeric.left_lt_right {x : pgame} (o : numeric x) (i : x.left_moves) (j : x.right_moves) :
x.move_left i < x.move_right j :=
by { cases x with xl xr xL xR, exact o.1 i j }
lemma numeric.move_left {x : pgame} (o : numeric x) (i : x.left_moves) :
numeric (x.move_left i) :=
begin
cases x with xl xr xL xR,
exact o.2.1 i,
end
by { cases x with xl xr xL xR, exact o.2.1 i }
lemma numeric.move_right {x : pgame} (o : numeric x) (j : x.right_moves) :
numeric (x.move_right j) :=
begin
cases x with xl xr xL xR,
exact o.2.2 j,
end
by { cases x with xl xr xL xR, exact o.2.2 j }

@[elab_as_eliminator]
theorem numeric_rec {C : pgame → Prop}
Expand Down

0 comments on commit 24bc2e1

Please sign in to comment.