mathlib3 documentation

data.real.golden_ratio

The golden ratio and its conjugate #

THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.

This file defines the golden ratio φ := (1 + √5)/2 and its conjugate ψ := (1 - √5)/2, which are the two real roots of X² - X - 1.

Along with various computational facts about them, we prove their irrationality, and we link them to the Fibonacci sequence by proving Binet's formula.

@[reducible]
noncomputable def golden_ratio  :

The golden ratio φ := (1 + √5)/2.

Equations
@[reducible]
noncomputable def golden_conj  :

The conjugate of the golden ratio ψ := (1 - √5)/2.

Equations

The inverse of the golden ratio is the opposite of its conjugate.

The opposite of the golden ratio is the inverse of its conjugate.

@[simp]
theorem gold_sq  :
@[simp]
theorem gold_pos  :

Irrationality #

The golden ratio is irrational.

The conjugate of the golden ratio is irrational.

def fib_rec {α : Type u_1} [comm_semiring α] :

The recurrence relation satisfied by the Fibonacci sequence.

Equations

The characteristic polynomial of fib_rec is X² - (X + 1).

theorem fib_is_sol_fib_rec {α : Type u_1} [comm_semiring α] :

As expected, the Fibonacci sequence is a solution of fib_rec.

The geometric sequence λ n, φ^n is a solution of fib_rec.

The geometric sequence λ n, ψ^n is a solution of fib_rec.

theorem real.coe_fib_eq'  :
(λ (n : ), (nat.fib n)) = λ (n : ), (golden_ratio ^ n - golden_conj ^ n) / 5

Binet's formula as a function equality.

theorem real.coe_fib_eq (n : ) :

Binet's formula as a dependent equality.