Skip to main content

Demostraciones de "f⁻¹(u ∩ v) = f⁻¹(u) ∩ f⁻¹(v)"


Demostrar con Lean4 y con Isabelle/HOL que

   f⁻¹(u  v) = f⁻¹(u)  f⁻¹(v)

Para ello, completar la siguiente teoría de Lean4:

import Mathlib.Data.Set.Function
variable {α β : Type _}
variable (f : α  β)
variable (u v : Set β)
open Set

example : f ⁻¹' (u  v) = f ⁻¹' u  f ⁻¹' v :=
by sorry

y la siguiente teoría de Iasbelle/HOL:

theory Imagen_inversa_de_la_interseccion
imports Main
begin

lemma "f -` (u ∩ v) = f -` u ∩ f -` v"
sorry

end

Read more…

Demostraciones de "s ∪ (⋂_i A_i) = ⋂_i (A_i ∪ s)"


Demostrar con Lean4 y con Isabelle/HOL que \[ s ∪ (⋂_i A_i) = ⋂_i (A_i ∪ s) \]

Para ello, completar la siguiente teoría de Lean4:

import Mathlib.Data.Set.Basic
import Mathlib.Tactic
open Set
variable {α : Type}
variable (s : Set α)
variable (A :   Set α)

example : s  ( i, A i) =  i, (A i  s) :=
by sorry

y la siguiente teoría de Isabelle/HOL:

theory Union_con_interseccion_general
imports Main
begin

lemma "s ∪ (⋂ i ∈ I. A i) = (⋂ i ∈ I. A i ∪ s)"
sorry

end

Read more…

Demostraciones de "⋂_i, (A(i) ∩ B(i)) = (⋂_i, A(i)) ∩ (⋂_i, B(i))"


Demostrar con Lean4 y con Isabelle/HOL que \[ ⋂_i (A_i ∩ B_i) = (⋂_i A_i) ∩ (⋂_i B_i) \]

Para ello, completar la siguiente teoría de Lean4:

import Mathlib.Data.Set.Basic
import Mathlib.Tactic

open Set

variable {α : Type}
variable (A B :   Set α)

example : ( i, A i  B i) = ( i, A i)  ( i, B i) :=
by sorry

la siguiente teoría de Isabelle/HOL:

theory Interseccion_de_intersecciones
imports Main
begin

lemma "(⋂ i ∈ I. A i ∩ B i) = (⋂ i ∈ I. A i) ∩ (⋂ i ∈ I. B i)"
sorry

end

Read more…

Demostraciones de "s ∩ ⋃_i A_i = ⋃_i (A_i ∩ s)"


Demostrar con Lean4 y con Isabelle/HOL que \[ s ∩ ⋃_i A_i = ⋃_i (A_i ∩ s) \]

Para ello, completar la siguiente teoría de Lean4:

import Mathlib.Data.Set.Basic
import Mathlib.Data.Set.Lattice
import Mathlib.Tactic

open Set

variable {α : Type}
variable (s : Set α)
variable (A :   Set α)

example : s  ( i, A i) =  i, (A i  s) :=
by sorry

y la siguiente teoría de Isabelle/HOL:

theory Distributiva_de_la_interseccion_respecto_de_la_union_general
imports Main
begin

lemma "s ∩ (⋃ i ∈ I. A i) = (⋃ i ∈ I. (A i ∩ s))"
sorry

end

Read more…

Los primos mayores que 2 son impares


Demostrar con Lean4 y con Isabelle/HOL que los primos mayores que 2 son impares. Para ello, completar la siguiente teoría de Lean4:

import Mathlib.Algebra.Ring.Parity
import Mathlib.Tactic

open Nat

def Primos      : Set  := {n | Nat.Prime n}
def MayoresQue2 : Set  := {n | n > 2}
def Impares     : Set  := {n | ¬Even n}

example : Primos  MayoresQue2  Impares :=
by sorry

y la siguiente teoría de Isabelle/HOL:

theory Interseccion_de_los_primos_y_los_mayores_que_dos
imports Main "HOL-Number_Theory.Number_Theory"
begin

definition primos :: "nat set" where
  "primos = {n ∈ ℕ . prime n}"

definition mayoresQue2 :: "nat set" where
  "mayoresQue2 = {n ∈ ℕ . n > 2}"

definition impares :: "nat set" where
  "impares = {n ∈ ℕ . ¬ even n}"

lemma "primos ∩ mayoresQue2 ⊆ impares"
oops

end

Read more…

La unión del conjunto de los números naturales pares e impares es el conjunto de los naturales


Demostrar con Lean4 y con Isabelle/HOL que la unión del conjunto de los números naturales pares e impares es el conjunto de los naturales. Para ello, completar la siguiente teoría de Lean4:

import Mathlib.Algebra.Ring.Parity

def Naturales : Set  := {n | True}
def Pares     : Set  := {n | Even n}
def Impares   : Set  := {n | ¬Even n}

example : Pares  Impares = Naturales :=
by sorry

y la siguiente teoría de Isabelle/HOL:

theory Union_de_pares_e_impares
imports Main
begin

definition naturales :: "nat set" where
  "naturales = {n ∈ ℕ . True}"

definition pares :: "nat set" where
  "pares = {n ∈ ℕ . even n}"

definition impares :: "nat set" where
  "impares = {n ∈ ℕ . ¬ even n}"

lemma "pares ∪ impares = naturales"
oops

end

Read more…

Demostraciones de "(s \ t) ∪ (t \ s) = (s ∪ t) \ (s ∩ t)"


Demostrar con Lean4 y con Isabelle/HOL que \[ (s \setminus t) ∪ (t \setminus s) = (s ∪ t) \setminus (s ∩ t) \]

Para ello, completar la siguiente teoría de Lean4:

import Mathlib.Data.Set.Basic
import Mathlib.Tactic

open Set

variable {α : Type}
variable (s t : Set α)

example : (s \\ t)  (t \\ s) = (s  t) \\ (s  t) :=
by sorry

y la siguiente teoría de Isabelle/HOL:

theory Diferencia_de_union_e_interseccion
imports Main
begin

lemma "(s - t) ∪ (t - s) = (s ∪ t) - (s ∩ t)"
oops

end

Read more…

Demostraciones de "(s \ t) ∪ t = s ∪ t"


Demostrar con Lean4 y con Isabelle/HOL que \[ (s \setminus t) ∪ t = s ∪ t \]

Para ello, completar la siguiente teoría de Lean4:

import Mathlib.Data.Set.Basic
open Set

variable {α : Type}
variable (s t : Set α)

example : (s \\setminus t)  t = s  t :=
by sorry

y la siguiente teoría de Isabelle/HOL:

theory Union_con_su_diferencia
imports Main
begin

lemma "(s - t) ∪ t = s ∪ t"
oops

end

Read more…

Demostraciones de "s ∪ (s ∩ t) = s"


Demostrar con Lean4 y con Isabelle/HOL que \[ s ∪ (s ∩ t) = s \]

Para ello, completar la siguiente teoría de Lean4:

import Mathlib.Data.Set.Basic
open Set
variable {α : Type}
variable (s t : Set α)

example : s  (s  t) = s :=
by sorry

y la siguiente teoría de Isabelle/HOL:

theory Union_con_su_interseccion
imports Main
begin

lemma "s ∪ (s ∩ t) = s"
oops

end

Read more…

Demostraciones de "s ∩ (s ∪ t) = s"


Demostrar con Lean4 y con Isabelle/HOL que \[ s ∩ (s ∪ t) = s \]

Para ello, completar la siguiente teoría de Lean4:

import Mathlib.Data.Set.Basic
import Mathlib.Tactic
open Set
variable {α : Type}
variable (s t : Set α)

example : s  (s  t) = s :=
by sorry

y la siguiente teoría de Isabelle/HOL:

theory Interseccion_con_su_union
imports Main
begin

lemma "s ∩ (s ∪ t) = s"
oops

wnd

Read more…