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

Commit 06f7d3f

Browse files
committed
feat(src/set_theory/surreal): add numeric_add and numeric_omega lemmas (#7179)
Adds a couple of lemmas about surreal numbers: proving that natural numbers and omega are numeric. [Zulip](https://leanprover.zulipchat.com/#narrow/stream/116395-maths/topic/Surreal.20numbers/near/234243582)
1 parent 46302c7 commit 06f7d3f

File tree

1 file changed

+8
-3
lines changed

1 file changed

+8
-3
lines changed

src/set_theory/surreal.lean

Lines changed: 8 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -253,9 +253,14 @@ theorem numeric_add : Π {x y : pgame} (ox : numeric x) (oy : numeric y), numeri
253253
end
254254
using_well_founded { dec_tac := pgame_wf_tac }
255255

256-
-- TODO prove
257-
-- theorem numeric_nat (n : ℕ) : numeric n := sorry
258-
-- theorem numeric_omega : numeric omega := sorry
256+
/-- Pre-games defined by natural numbers are numeric. -/
257+
theorem numeric_nat : Π (n : ℕ), numeric n
258+
| 0 := numeric_zero
259+
| (n + 1) := numeric_add (numeric_nat n) numeric_one
260+
261+
/-- The pre-game omega is numeric. -/
262+
theorem numeric_omega : numeric omega :=
263+
by rintros ⟨⟩ ⟨⟩, λ i, numeric_nat i.down, by rintros ⟨⟩⟩
259264

260265
end pgame
261266

0 commit comments

Comments
 (0)