-
Notifications
You must be signed in to change notification settings - Fork 1
/
Copy pathFunciones_no_monotonas.lean
70 lines (56 loc) · 1.77 KB
/
Funciones_no_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
-- ---------------------------------------------------------------------
-- Ejercicio 1. Realizar las siguientes acciones:
-- 1. Importar la teoría de los números reales.
-- 2. Declarar f como una variable sobre las funciones de ℝ en ℝ.
-- ----------------------------------------------------------------------
import data.real.basic -- 1
variable {f : ℝ → ℝ} -- 2
-- ---------------------------------------------------------------------
-- Ejercicio 2. Demostrar que f es no monótona syss existen x e y tales
-- que x ≤ y y f(x) > f(y).
-- ----------------------------------------------------------------------
-- 1ª demostración
-- ================
example :
¬ monotone f ↔ ∃ x y, x ≤ y ∧ f x > f y :=
begin
rw [monotone],
push_neg,
end
-- Prueba
-- ======
/-
f : ℝ → ℝ
⊢ ¬monotone f ↔ ∃ (x y : ℝ), x ≤ y ∧ f x > f y
>> rw [monotone],
⊢ (¬∀ ⦃a b : ℝ⦄, a ≤ b → f a ≤ f b) ↔ ∃ (x y : ℝ), x ≤ y ∧ f x > f y
>> push_neg,
no goals
-/
-- Comentario: Se ha usado la definición
-- + monotone: ∀ ⦃a b : ℝ⦄, a ≤ b → f a ≤ f b
-- 2ª demostración
-- ================
lemma not_monotone_iff :
¬ monotone f ↔ ∃ x y, x ≤ y ∧ f x > f y :=
by { rw [monotone], push_neg }
-- ---------------------------------------------------------------------
-- Ejercicio 3. Demostrar que la función opuesta no es monótona.
-- ----------------------------------------------------------------------
example : ¬ monotone (λ x : ℝ, -x) :=
begin
apply not_monotone_iff.mpr,
use [2, 3],
norm_num,
end
-- Prueba
-- ======
/-
⊢ ¬monotone (λ (x : ℝ), -x)
>> apply not_monotone_iff.mpr,
⊢ ∃ (x y : ℝ), x ≤ y ∧ -x > -y
>> use [2, 3],
⊢ 2 ≤ 3 ∧ -2 > -3
>> norm_num,
no goals
-/