-
Notifications
You must be signed in to change notification settings - Fork 1
/
two_mul.lean
33 lines (27 loc) · 1.13 KB
/
two_mul.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
-- ---------------------------------------------------------------------
-- Ejercicio 1. Realizar las siguientes acciones:
-- 1. Importar la teoría de anillos.
-- 2. Crear el espacio de nombres my_ring
-- 3. Declarar R como una variable sobre anillos.
-- 4. Declarar a como variable sobre R.
-- ----------------------------------------------------------------------
import algebra.ring -- 1
namespace my_ring -- 2
variables {R : Type*} [ring R] -- 3
variables (a : R) -- 4
-- ---------------------------------------------------------------------
-- Ejercicio 2. Demostrar que
-- 1 + 1 = 2
-- ----------------------------------------------------------------------
lemma one_add_one_eq_two : 1 + 1 = (2 : R) :=
by refl
-- ---------------------------------------------------------------------
-- Ejercicio 3. Demostrar que
-- 2 * a = a + a
-- ----------------------------------------------------------------------
theorem two_mul : 2 * a = a + a :=
calc
2 * a = (1 + 1) * a : by rw one_add_one_eq_two
... = 1 * a + 1 * a : by rw add_mul
... = a + a : by rw one_mul
end my_ring