-
Notifications
You must be signed in to change notification settings - Fork 1
/
Copy pathComposicion_de_funciones_monotonas.lean
64 lines (55 loc) · 1.33 KB
/
Composicion_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
-- ---------------------------------------------------------------------
-- Ejercicio. Demostrar que la composición de dos funciones monótonas es
-- monótona.
-- ----------------------------------------------------------------------
import data.real.basic
variables (f g : ℝ → ℝ)
-- 1ª demostración
-- ===============
example
(mf : monotone f)
(mg : monotone g)
: monotone (f ∘ g) :=
begin
have h1 : ∀ a b, a ≤ b → (f ∘ g) a ≤ (f ∘ g) b,
{ intros a b hab,
have h1 : g a ≤ g b := mg hab,
have h2 : f (g a) ≤ f (g b) := mf h1,
show (f ∘ g) a ≤ (f ∘ g) b,
by exact h2, },
show monotone (f ∘ g),
by exact h1,
end
-- 2ª demostración
-- ===============
example
(mf : monotone f)
(mg : monotone g)
: monotone (f ∘ g) :=
begin
intros a b hab,
apply mf,
apply mg,
apply hab
end
-- Su desarrollo es
--
-- f g : ℝ → ℝ,
-- mf : monotone f,
-- mg : monotone g
-- ⊢ monotone (λ (x : ℝ), f (g x))
-- >> intros a b hab,
-- a b : ℝ,
-- hab : a ≤ b
-- ⊢ (λ (x : ℝ), f (g x)) a ≤ (λ (x : ℝ), f (g x)) b
-- >> apply mf,
-- ⊢ g a ≤ g b
-- >> apply mg,
-- ⊢ a ≤ b
-- >> apply hab
-- no goals
-- 3ª demostración
-- ===============
example (mf : monotone f) (mg : monotone g) :
monotone (f ∘ g) :=
λ a b hab, mf (mg hab)