-
Notifications
You must be signed in to change notification settings - Fork 1
/
Copy pathAnillos_ordenados.lean
29 lines (25 loc) · 1.14 KB
/
Anillos_ordenados.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
-- ---------------------------------------------------------------------
-- Ejercicio 1. Realizar las siguientes acciones
-- 1. Importar la teoría de los anillos ordenados.
-- 2. Declarar R como un tipo sobre los anillos ordenados.
-- 3. Declarar a y b como variables sobre R.
-- ----------------------------------------------------------------------
import algebra.ordered_ring -- 1
variables {R : Type*} [ordered_ring R] -- 2
variables a b : R -- 3
-- ---------------------------------------------------------------------
-- Ejercicio 2. Calcular el tipo de las siguientes expresiones
-- @add_le_add_left R _ a b
-- @mul_pos R _ a b
-- zero_ne_one
-- @mul_nonneg R _ a b
-- ----------------------------------------------------------------------
-- #check @add_le_add_left
-- #check @mul_pos R _ a b
-- #check zero_ne_one
-- #check @mul_nonneg R _ a b
-- Comentario: Al colocar el cursor sobre check se obtiene
-- add_le_add_left : a ≤ b → ∀ c, c + a ≤ c + b
-- mul_pos : 0 < a → 0 < b → 0 < a * b
-- zero_ne_one : 0 ≠ 1
-- mul_nonneg : 0 ≤ a → 0 ≤ b → 0 ≤ a * b