Para todo c ∈ ℝ, la función f(x) = x+c es inyectiva
Demostrar que para todo c ∈ ℝ, la función f(x) = x+c es inyectiva.
Para ello, completar la siguiente teoría de Lean:
1 2 3 4 5 6 7 8 |
import data.real.basic open function variable {c : ℝ} example : injective (λ x, x + c) := sorry |
Soluciones con Lean
1 2 3 4 5 6 7 8 9 10 11 12 13 14 15 16 17 18 19 20 21 22 23 24 25 26 27 28 29 30 31 32 33 34 35 36 37 38 39 40 41 42 43 |
import data.real.basic open function variable {c : ℝ} -- 1ª demostración -- =============== example : injective (λ x, x + c) := begin assume x1 : ℝ, assume x2 : ℝ, assume h1 : (λ x, x + c) x1 = (λ x, x + c) x2, have h2 : x1 + c = x2 + c := h1, show x1 = x2, by exact (add_left_inj c).mp h2, end -- 2ª demostración -- =============== example : injective (λ x, x + c) := begin intros x1 x2 h, change x1 + c = x2 + c at h, apply add_right_cancel h, end -- 3ª demostración -- =============== example : injective (λ x, x + c) := begin intros x1 x2 h, apply (add_left_inj c).mp, exact h, end -- 4ª demostración -- =============== example : injective (λ x, x + c) := λ x1 x2 h, (add_left_inj c).mp h |
Se puede interactuar con la prueba anterior en esta sesión con Lean.
Referencias
- J. Avigad, K. Buzzard, R.Y. Lewis y P. Massot. Mathematics in Lean, p. 29.