mathlib3 documentation

set_theory.surreal.dyadic

Dyadic numbers #

THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4. Dyadic numbers are obtained by localizing ℤ away from 2. They are the initial object in the category of rings with no 2-torsion.

Dyadic surreal numbers #

We construct dyadic surreal numbers using the canonical map from ℤ[2 ^ {-1}] to surreals. As we currently do not have a ring structure on surreal we construct this map explicitly. Once we have the ring structure, this map can be constructed directly by sending 2 ^ {-1} to half.

Embeddings #

The above construction gives us an abelian group embedding of ℤ into surreal. The goal is to extend this to an embedding of dyadic rationals into surreal and use Cauchy sequences of dyadic rational numbers to construct an ordered field embedding of ℝ into surreal.

For a natural number n, the pre-game pow_half (n + 1) is recursively defined as {0 | pow_half n}. These are the explicit expressions of powers of 1 / 2. By definition, we have pow_half 0 = 1 and pow_half 1 ≈ 1 / 2 and we prove later on that pow_half (n + 1) + pow_half (n + 1) ≈ pow_half n.

Equations
@[simp]
@[simp]

For all natural numbers n, the pre-games pow_half n are numeric.

Powers of the surreal number half.

Equations
@[simp]
theorem surreal.zsmul_pow_two_pow_half (m : ) (n k : ) :
theorem surreal.dyadic_aux {m₁ m₂ : } {y₁ y₂ : } (h₂ : m₁ * 2 ^ y₁ = m₂ * 2 ^ y₂) :

The additive monoid morphism dyadic_map sends ⟦⟨m, 2^n⟩⟧ to m • half ^ n.

Equations

We define dyadic surreals as the range of the map dyadic_map.

Equations