Las familias de conjuntos definen relaciones simétricas
Cada familia de conjuntos P define una relación de forma que dos elementos están relacionados si algún conjunto de P contiene a ambos elementos. Se puede definir en Lean por
1 2 |
def relacion (P : set (set X)) (x y : X) := ∃ A ∈ P, x ∈ A ∧ y ∈ A |
Demostrar que si P es una familia de subconjunt❙os de X, entonces la relación definida por P es simétrica.
Para ello, completar la siguiente teoría de Lean:
1 2 3 4 5 6 7 8 9 10 |
import tactic variable {X : Type} variable (P : set (set X)) def relacion (P : set (set X)) (x y : X) := ∃ A ∈ P, x ∈ A ∧ y ∈ A example : symmetric (relacion P) := sorry |
[expand title=»Soluciones con 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 |
import tactic variable {X : Type} variable (P : set (set X)) def relacion (P : set (set X)) (x y : X) := ∃ A ∈ P, x ∈ A ∧ y ∈ A -- 1ª demostración example : symmetric (relacion P) := begin unfold symmetric, intros x y hxy, unfold relacion at *, rcases hxy with ⟨B, hBP, ⟨hxB, hyB⟩⟩, use B, repeat { split }, { exact hBP, }, { exact hyB, }, { exact hxB, }, end -- 2ª demostración example : symmetric (relacion P) := begin intros x y hxy, rcases hxy with ⟨B, hBP, ⟨hxB, hyB⟩⟩, use B, repeat { split } ; assumption, end -- 3ª demostración example : symmetric (relacion P) := begin intros x y hxy, rcases hxy with ⟨B, hBP, ⟨hxB, hyB⟩⟩, use [B, ⟨hBP, hyB, hxB⟩], end |
Se puede interactuar con la prueba anterior en esta sesión con Lean.
En los comentarios se pueden escribir otras soluciones, escribiendo el código entre una línea con <pre lang="lean"> y otra con </pre>
[/expand]
[expand title=»Soluciones con Isabelle/HOL»]
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 |
theory Las_familias_de_conjuntos_definen_relaciones_simetricas imports Main begin definition relacion :: "('a set) set ⇒ 'a ⇒ 'a ⇒ bool" where "relacion P x y ⟷ (∃A∈P. x ∈ A ∧ y ∈ A)" (* 1ª demostración *) lemma "symp (relacion P)" proof (rule sympI) fix x y assume "relacion P x y" then have "∃A∈P. x ∈ A ∧ y ∈ A" by (unfold relacion_def) then have "∃A∈P. y ∈ A ∧ x ∈ A" proof (rule bexE) fix A assume hA1 : "A ∈ P" and hA2 : "x ∈ A ∧ y ∈ A" have "y ∈ A ∧ x ∈ A" using hA2 by (simp only: conj_commute) then show "∃A∈P. y ∈ A ∧ x ∈ A" using hA1 by (rule bexI) qed then show "relacion P y x" by (unfold relacion_def) qed (* 2ª demostración *) lemma "symp (relacion P)" proof (rule sympI) fix x y assume "relacion P x y" then obtain A where "A ∈ P ∧ x ∈ A ∧ y ∈ A" using relacion_def by metis then show "relacion P y x" using relacion_def by metis qed (* 3ª demostración *) lemma "symp (relacion P)" using relacion_def by (metis sympI) end |
En los comentarios se pueden escribir otras soluciones, escribiendo el código entre una línea con <pre lang="isar"> y otra con </pre>
[/expand]