-
Notifications
You must be signed in to change notification settings - Fork 1
/
Propiedades_de_funciones_monotonas.lean
83 lines (74 loc) · 1.78 KB
/
Propiedades_de_funciones_monotonas.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
66
67
68
69
70
71
72
73
74
75
76
77
78
79
80
81
82
83
-- ---------------------------------------------------------------------
-- Ejercicio 1. Realizar las siguientes acciones
-- 1. Importar la librería de los reales.
-- 2. Declarar f como variable de las funciones de ℝ en ℝ.
-- 3. Declarar a y b como variables sobre los reales.
-- ----------------------------------------------------------------------
import data.real.basic -- 1
variables (f : ℝ → ℝ) -- 2
variables (a b : ℝ) -- 3
-- ---------------------------------------------------------------------
-- Ejercicio 2. Demostrar que si f es monótona y f(a) < f(b), entonces
-- a < b
-- ----------------------------------------------------------------------
example
(h : monotone f)
(h' : f a < f b)
: a < b :=
begin
apply lt_of_not_ge,
intro hab,
have : f a ≥ f b,
from h hab,
linarith,
end
-- Prueba
-- ======
-- f : ℝ → ℝ,
-- a b : ℝ,
-- h : monotone f,
-- h' : f a < f b
-- ⊢ a < b
-- >> apply lt_of_not_ge,
-- ⊢ ¬a ≥ b
-- >> intro hab,
-- hab : a ≥ b
-- ⊢ false
-- >> have : f a ≥ f b,
-- >> from h hab,
-- this : f a ≥ f b
-- ⊢ false
-- >> linarith,
-- no goals
-- ---------------------------------------------------------------------
-- Ejercicio 3. Demostrar que si
-- a ≤ b
-- f b < f a
-- entonces f no es monótona.
-- ----------------------------------------------------------------------
example
(h : a ≤ b)
(h' : f b < f a)
: ¬ monotone f :=
begin
intro h1,
have : f a ≤ f b,
from h1 h,
linarith,
end
-- Prueba
-- ======
-- f : ℝ → ℝ,
-- a b : ℝ,
-- h : a ≤ b,
-- h' : f b < f a
-- ⊢ ¬monotone f
-- >> intro h1,
-- h1 : monotone f
-- ⊢ false
-- >> have : f a ≤ f b,
-- >> from h1 h,
-- this : f a ≤ f b
-- ⊢ false
-- >> linarith,
-- no goals