-
Notifications
You must be signed in to change notification settings - Fork 0
/
Copy pathInecuaciones_con_exponenciales_4.lean
65 lines (52 loc) · 1.56 KB
/
Inecuaciones_con_exponenciales_4.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
44
45
46
47
48
49
50
51
52
53
54
55
56
57
58
59
60
61
62
63
64
65
-- Inecuaciones_con_exponenciales_4.lean
-- En ℝ, si a ≤ b, entonces c - e^b ≤ c - e^a.
-- José A. Alonso Jiménez <https://jaalonso.github.io>
-- Sevilla, 31-agosto-2023
-- ---------------------------------------------------------------------
-- ---------------------------------------------------------------------
-- Sean a, b y c números reales. Demostrar que si
-- a ≤ b
-- entonces
-- c - e^b ≤ c - e^a
-- ----------------------------------------------------------------------
-- Demostración en lenguaje natural
-- ================================
-- Aplicando la monotonía de la exponencial a la hipótesis, se tiene
-- e^a ≤ e^b
-- y, restando de c, se invierte la desigualdad
-- c - e^b ≤ c - e^a
-- Demostraciones con Lean4
-- ========================
import Mathlib.Analysis.SpecialFunctions.Log.Basic
open Real
variable (a b c : ℝ)
-- 1ª demostración
example
(h : a ≤ b)
: c - exp b ≤ c - exp a :=
by
have h1 : exp a ≤ exp b :=
exp_le_exp.mpr h
show c - exp b ≤ c - exp a
exact sub_le_sub_left h1 c
-- 2ª demostración
example
(h : a ≤ b)
: c - exp b ≤ c - exp a :=
by
apply sub_le_sub_left _ c
apply exp_le_exp.mpr h
-- 3ª demostración
example
(h : a ≤ b)
: c - exp b ≤ c - exp a :=
sub_le_sub_left (exp_le_exp.mpr h) c
-- 4ª demostración
example
(h : a ≤ b)
: c - exp b ≤ c - exp a :=
by linarith [exp_le_exp.mpr h]
-- Lemas usados
-- ============
-- #check (exp_le_exp : exp a ≤ exp b ↔ a ≤ b)
-- #check (sub_le_sub_left : a ≤ b → ∀ (c : ℝ), c - b ≤ c - a)