-
Notifications
You must be signed in to change notification settings - Fork 1
/
Copy pathLas_tacticas_apply_y_exact.lean
101 lines (84 loc) · 1.85 KB
/
Las_tacticas_apply_y_exact.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
84
85
86
87
88
89
90
91
92
93
94
95
96
97
98
99
100
101
-- ---------------------------------------------------------------------
-- Ejercicio 1. Realizar las siguientes acciones:
-- 1. Importar la teoría de los números reales
-- 2. Declarar x, y y z como variables sobre R.
-- ----------------------------------------------------------------------
import data.real.basic
variables (x y z : ℝ)
-- ---------------------------------------------------------------------
-- Ejercicio 2. Demostrar que si
-- x ≤ y
-- y ≤ z
-- entonces
-- x ≤ z
-- ----------------------------------------------------------------------
-- 1ª demostración
-- ===============
example
(h1 : x ≤ y)
(h2 : y ≤ z)
: x ≤ z :=
begin
apply le_trans,
{ apply h1, },
apply h2,
end
-- El desarrollo de la prueba es
--
-- x y z : ℝ,
-- h1 : x ≤ y,
-- h2 : y ≤ z
-- ⊢ x ≤ z
-- apply le_trans,
-- ⊢ x ≤ ?m_1
-- { apply h1 },
-- ⊢ y ≤ z
-- apply h2,
-- no goals
-- 2ª demostración
-- ===============
example
(h1 : x ≤ y)
(h2 : y ≤ z)
: x ≤ z :=
begin
apply le_trans h1,
apply h2,
end
-- El desarrollo de la prueba es
--
-- x y z : ℝ,
-- h1 : x ≤ y,
-- h2 : y ≤ z
-- ⊢ x ≤ z
-- apply le_trans h1,
-- ⊢ y ≤ z
-- apply h2,
-- no goals
-- 3ª demostración
-- ===============
example
(h1 : x ≤ y)
(h2 : y ≤ z)
: x ≤ z :=
by exact le_trans h1 h2
-- 4ª demostración
-- ===============
example
(h1 : x ≤ y)
(h2 : y ≤ z)
: x ≤ z :=
le_trans h1 h2
-- ---------------------------------------------------------------------
-- Ejercicio 4. Demostrar que
-- x ≤ x
-- ----------------------------------------------------------------------
-- 1ª demostración
example : x ≤ x :=
by apply le_refl
-- 2ª demostración
example : x ≤ x :=
by exact le_refl x
-- 3ª demostración
example (x : ℝ) : x ≤ x :=
le_refl x