mathlib documentation

data.​real.​basic

data.​real.​basic

def real  :
Type

Equations
@[instance]

Equations
@[instance]

Equations
@[instance]

Equations

Coercion as a ring_hom. Note that this is cau_seq.completion.of_rat, not rat.cast.

Equations
def real.​mk  :

Make a real number from a Cauchy sequence of rationals (by taking the equivalence class).

Equations
@[instance]

Equations
@[simp]
theorem real.​mk_lt {f g : cau_seq abs} :

theorem real.​mk_eq {f g : cau_seq abs} :

@[simp]
theorem real.​mk_pos {f : cau_seq abs} :

def real.​le  :
→ Prop

Equations
@[instance]

Equations
@[simp]
theorem real.​mk_le {f g : cau_seq abs} :

theorem real.​add_lt_add_iff_left {a b : } (c : ) :
c + a < c + b a < b

@[instance]

Equations
theorem real.​zero_lt_one  :
0 < 1

theorem real.​mul_pos {a b : } :
0 < a0 < b0 < a * b

@[instance]

Equations
@[instance]

Equations
@[instance]
def real.​decidable_lt (a b : ) :
decidable (a < b)

Equations
@[instance]
def real.​decidable_le (a b : ) :

Equations
@[instance]
def real.​decidable_eq (a b : ) :
decidable (a = b)

Equations
theorem real.​le_of_forall_epsilon_le {a b : } :
(∀ (ε : ), 0 < εa b + ε)a b

@[simp]

theorem real.​le_mk_of_forall_le {x : } {f : cau_seq abs} :
(∃ (i : ), ∀ (j : ), j ix (f j))x real.mk f

theorem real.​mk_le_of_forall_le {f : cau_seq abs} {x : } :
(∃ (i : ), ∀ (j : ), j i(f j) x)real.mk f x

theorem real.​mk_near_of_forall_near {f : cau_seq abs} {x ε : } :
(∃ (i : ), ∀ (j : ), j iabs ((f j) - x) ε)abs (real.mk f - x) ε

@[instance]

Equations
theorem real.​is_cau_seq_iff_lift {f : } :
is_cau_seq abs f is_cau_seq abs (λ (i : ), (f i))

theorem real.​of_near (f : ) (x : ) :
(∀ (ε : ), ε > 0(∃ (i : ), ∀ (j : ), j iabs ((f j) - x) < ε))(∃ (h' : is_cau_seq abs f), real.mk f, h'⟩ = x)

theorem real.​exists_floor (x : ) :
∃ (ub : ), ub x ∀ (z : ), z xz ub

theorem real.​exists_sup (S : set ) :
(∃ (x : ), x S)(∃ (x : ), ∀ (y : ), y Sy x)(∃ (x : ), ∀ (y : ), x y ∀ (z : ), z Sz y)

@[instance]

Equations
theorem real.​Sup_def (S : set ) :
has_Sup.Sup S = dite ((∃ (x : ), x S) ∃ (x : ), ∀ (y : ), y Sy x) (λ (h : (∃ (x : ), x S) ∃ (x : ), ∀ (y : ), y Sy x), classical.some _) (λ (h : ¬((∃ (x : ), x S) ∃ (x : ), ∀ (y : ), y Sy x)), 0)

theorem real.​Sup_le (S : set ) (h₁ : ∃ (x : ), x S) (h₂ : ∃ (x : ), ∀ (y : ), y Sy x) {y : } :
has_Sup.Sup S y ∀ (z : ), z Sz y

theorem real.​lt_Sup (S : set ) (h₁ : ∃ (x : ), x S) (h₂ : ∃ (x : ), ∀ (y : ), y Sy x) {y : } :
y < has_Sup.Sup S ∃ (z : ) (H : z S), y < z

theorem real.​le_Sup (S : set ) (h₂ : ∃ (x : ), ∀ (y : ), y Sy x) {x : } :
x Sx has_Sup.Sup S

theorem real.​Sup_le_ub (S : set ) (h₁ : ∃ (x : ), x S) {ub : } :
(∀ (y : ), y Sy ub)has_Sup.Sup S ub

theorem real.​is_lub_Sup {s : set } {a b : } :
a sb upper_bounds sis_lub s (has_Sup.Sup s)

@[instance]

Equations
theorem real.​Inf_def (S : set ) :

theorem real.​le_Inf (S : set ) (h₁ : ∃ (x : ), x S) (h₂ : ∃ (x : ), ∀ (y : ), y Sx y) {y : } :
y has_Inf.Inf S ∀ (z : ), z Sy z

theorem real.​Inf_lt (S : set ) (h₁ : ∃ (x : ), x S) (h₂ : ∃ (x : ), ∀ (y : ), y Sx y) {y : } :
has_Inf.Inf S < y ∃ (z : ) (H : z S), z < y

theorem real.​Inf_le (S : set ) (h₂ : ∃ (x : ), ∀ (y : ), y Sx y) {x : } :
x Shas_Inf.Inf S x

theorem real.​lb_le_Inf (S : set ) (h₁ : ∃ (x : ), x S) {lb : } :
(∀ (y : ), y Slb y)lb has_Inf.Inf S

theorem real.​sqrt_exists {x : } :
0 x(∃ (y : ), 0 y y * y = x)

Equations
def real.​sqrt  :

The square root of a real number. This returns 0 for negative inputs.

Equations
theorem real.​sqrt_eq_zero_of_nonpos {x : } :
x 0real.sqrt x = 0

theorem real.​sqrt_nonneg (x : ) :

@[simp]
theorem real.​mul_self_sqrt {x : } :
0 xreal.sqrt x * real.sqrt x = x

@[simp]
theorem real.​sqrt_mul_self {x : } :
0 xreal.sqrt (x * x) = x

theorem real.​sqrt_eq_iff_mul_self_eq {x y : } :
0 x0 y(real.sqrt x = y y * y = x)

@[simp]
theorem real.​sqr_sqrt {x : } :
0 xreal.sqrt x ^ 2 = x

@[simp]
theorem real.​sqrt_sqr {x : } :
0 xreal.sqrt (x ^ 2) = x

theorem real.​sqrt_eq_iff_sqr_eq {x y : } :
0 x0 y(real.sqrt x = y y ^ 2 = x)

theorem real.​sqrt_sqr_eq_abs (x : ) :
real.sqrt (x ^ 2) = abs x

@[simp]
theorem real.​sqrt_zero  :

@[simp]
theorem real.​sqrt_one  :

@[simp]
theorem real.​sqrt_le {x y : } :
0 x0 y(real.sqrt x real.sqrt y x y)

@[simp]
theorem real.​sqrt_lt {x y : } :
0 x0 y(real.sqrt x < real.sqrt y x < y)

theorem real.​sqrt_le_sqrt {x y : } :

theorem real.​sqrt_le_left {x y : } :
0 y(real.sqrt x y x y ^ 2)

theorem real.​le_sqrt {x y : } :
0 x0 y(x real.sqrt y x ^ 2 y)

theorem real.​le_sqrt' {x y : } :
0 < x(x real.sqrt y x ^ 2 y)

theorem real.​le_sqrt_of_sqr_le {x y : } :
x ^ 2 yx real.sqrt y

@[simp]
theorem real.​sqrt_inj {x y : } :
0 x0 y(real.sqrt x = real.sqrt y x = y)

@[simp]
theorem real.​sqrt_eq_zero {x : } :
0 x(real.sqrt x = 0 x = 0)

theorem real.​sqrt_eq_zero' {x : } :
real.sqrt x = 0 x 0

@[simp]
theorem real.​sqrt_pos {x : } :
0 < real.sqrt x 0 < x

@[simp]
theorem real.​sqrt_mul' (x : ) {y : } :
0 yreal.sqrt (x * y) = real.sqrt x * real.sqrt y

@[simp]
theorem real.​sqrt_mul {x : } (hx : 0 x) (y : ) :

@[simp]

@[simp]
theorem real.​sqrt_div {x : } (hx : 0 x) (y : ) :