Skip to content

Commit

Permalink
feat(set_theory/ordinal/basic): rel_iso.ordinal_type_eq (#14602)
Browse files Browse the repository at this point in the history
  • Loading branch information
vihdzp committed Jun 8, 2022
1 parent 09df85f commit 8934884
Showing 1 changed file with 4 additions and 0 deletions.
4 changes: 4 additions & 0 deletions src/set_theory/ordinal/basic.lean
Expand Up @@ -504,6 +504,10 @@ theorem type_eq {α β} {r : α → α → Prop} {s : β → β → Prop}
[is_well_order α r] [is_well_order β s] :
type r = type s ↔ nonempty (r ≃r s) := quotient.eq

theorem _root_.rel_iso.ordinal_type_eq {α β} {r : α → α → Prop} {s : β → β → Prop}
[is_well_order α r] [is_well_order β s] (h : r ≃r s) :
type r = type s := type_eq.2 ⟨h⟩

@[simp] theorem type_lt (o : ordinal) : type ((<) : o.out.α → o.out.α → Prop) = o :=
begin
change type o.out.r = _,
Expand Down

0 comments on commit 8934884

Please sign in to comment.