Skip to content

Commit

Permalink
feat(set_theory/zfc/basic): better docs on univ_not_mem_univ (#18234)
Browse files Browse the repository at this point in the history
This theorem is somewhat odd, but phrases a very important result: there is no ZFC universal set. The new docs better clarify this.
  • Loading branch information
vihdzp committed Jan 22, 2023
1 parent 831c494 commit 800d3d4
Showing 1 changed file with 4 additions and 1 deletion.
5 changes: 4 additions & 1 deletion src/set_theory/zfc/basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -894,7 +894,10 @@ instance : is_asymm Class (∈) := mem_wf.is_asymm
theorem mem_asymm {x y : Class} : x ∈ y → y ∉ x := asymm
theorem mem_irrefl (x : Class) : x ∉ x := irrefl x

/-- There is no universal set. -/
/-- **There is no universal set.**
This is stated as `univ ∉ univ`, meaning that `univ` (the class of all sets) is proper (does not
belong to the class of all sets). -/
theorem univ_not_mem_univ : univ ∉ univ := mem_irrefl _

/-- Convert a conglomerate (a collection of classes) into a class -/
Expand Down

0 comments on commit 800d3d4

Please sign in to comment.