Skip to content

Commit

Permalink
feat(set_theory/zfc): basic lemmas on pSet.equiv (#15211)
Browse files Browse the repository at this point in the history
We unfold the complex definition into something easier to use.
  • Loading branch information
vihdzp committed Jul 10, 2022
1 parent 4b6ec60 commit cf4783f
Showing 1 changed file with 8 additions and 0 deletions.
8 changes: 8 additions & 0 deletions src/set_theory/zfc.lean
Expand Up @@ -98,6 +98,14 @@ equivalent to some element of the second family and vice-versa. -/
def equiv (x y : pSet) : Prop :=
pSet.rec (λ α z m ⟨β, B⟩, (∀ a, ∃ b, m a (B b)) ∧ (∀ b, ∃ a, m a (B b))) x y

theorem exists_equiv_left : Π {x y : pSet} (h : equiv x y) (i : x.type),
∃ j, equiv (x.func i) (y.func j)
| ⟨α, A⟩ ⟨β, B⟩ h := h.1

theorem exists_equiv_right : Π {x y : pSet} (h : equiv x y) (j : y.type),
∃ i, equiv (x.func i) (y.func j)
| ⟨α, A⟩ ⟨β, B⟩ h := h.2

theorem equiv.refl (x) : equiv x x :=
pSet.rec_on x $ λ α A IH, ⟨λ a, ⟨a, IH a⟩, λ a, ⟨a, IH a⟩⟩

Expand Down

0 comments on commit cf4783f

Please sign in to comment.