Skip to content

Commit

Permalink
feat(set_theory/ordinal): Small iff cardinality less than `cardinal.u…
Browse files Browse the repository at this point in the history
…niv` (#12887)

Characterizes when a type is small in terms of its cardinality
  • Loading branch information
awainverse committed Mar 22, 2022
1 parent 3838b85 commit d711d2a
Show file tree
Hide file tree
Showing 2 changed files with 13 additions and 1 deletion.
13 changes: 13 additions & 0 deletions src/set_theory/ordinal.lean
Expand Up @@ -4,6 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Mario Carneiro, Floris van Doorn
-/
import data.sum.order
import logic.small
import order.succ_pred.basic
import set_theory.cardinal

Expand Down Expand Up @@ -1385,6 +1386,18 @@ theorem lt_univ' {c} : c < univ.{u v} ↔ ∃ c', c = lift.{(max (u+1) v) u} c'
exact ⟨c', by simp only [e.symm, lift_lift]⟩
end, λ ⟨c', e⟩, e.symm ▸ lift_lt_univ' _⟩

theorem small_iff_lift_mk_lt_univ {α : Type u} :
small.{v} α ↔
(cardinal.lift (# α : cardinal.{u}) < univ.{v (max u (v + 1))}) :=
begin
rw lt_univ',
split,
{ rintro ⟨β, e⟩,
exact ⟨# β, (lift_mk_eq.{u _ (v + 1)}.2 e)⟩ },
{ rintro ⟨c, hc⟩,
exact ⟨⟨c.out, lift_mk_eq.{u _ (v + 1)}.1 (hc.trans (congr rfl c.mk_out.symm))⟩⟩ }
end

end cardinal

namespace ordinal
Expand Down
1 change: 0 additions & 1 deletion src/set_theory/ordinal_arithmetic.lean
Expand Up @@ -3,7 +3,6 @@ Copyright (c) 2017 Johannes Hölzl. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Mario Carneiro, Floris van Doorn, Violeta Hernández Palacios
-/
import logic.small
import set_theory.ordinal
import tactic.by_contra

Expand Down

0 comments on commit d711d2a

Please sign in to comment.