bookshelf/Bookshelf/Enderton/Set/Chapter_3.lean

22 lines
557 B
Plaintext
Raw Normal View History

2023-06-07 02:16:06 +00:00
import Mathlib.Data.Set.Basic
2023-06-08 23:57:02 +00:00
import Mathlib.SetTheory.ZFC.Basic
import Common.Set.OrderedPair
2023-06-07 02:16:06 +00:00
/-! # Enderton.Chapter_3
Relations and Functions
-/
namespace Enderton.Set.Chapter_3
2023-06-08 23:57:02 +00:00
/--
If `x ∈ C` and `y ∈ C`, then `⟨x, y⟩ ∈ 𝒫 𝒫 C`.
-/
theorem theorem_3b {C : Set α} (hx : x ∈ C) (hy : y ∈ C)
: Set.OrderedPair x y ∈ 𝒫 𝒫 C := by
have hxs : {x} ⊆ C := Set.singleton_subset_iff.mpr hx
have hxys : {x, y} ⊆ C := Set.mem_mem_imp_pair_subset hx hy
exact Set.mem_mem_imp_pair_subset hxs hxys
2023-06-07 02:16:06 +00:00
end Enderton.Set.Chapter_3