Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit 5931c5c

Browse files
committed
lint(set_theory/ordinal): fix def/lemma (#6369)
1 parent 3c66fd1 commit 5931c5c

File tree

1 file changed

+3
-4
lines changed

1 file changed

+3
-4
lines changed

src/set_theory/ordinal.lean

Lines changed: 3 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -1129,10 +1129,9 @@ begin
11291129
exact ordinal.min_le (λ i:ι α, ⟦⟨α, i.1, i.2⟩⟧) ⟨_, _⟩
11301130
end
11311131

1132-
@[nolint def_lemma doc_blame]
1133-
-- TODO: This should be a theorem but Lean fails to synthesize the placeholder
1134-
def ord_eq_min (α : Type u) : ord (mk α) =
1135-
@ordinal.min _ _ (λ i:{r // is_well_order α r}, ⟦⟨α, i.1, i.2⟩⟧) := rfl
1132+
lemma ord_eq_min (α : Type u) : ord (mk α) =
1133+
@ordinal.min {r // is_well_order α r} ⟨⟨well_ordering_rel, by apply_instance⟩⟩
1134+
(λ i, ⟦⟨α, i.1, i.2⟩⟧) := rfl
11361135

11371136
theorem ord_eq (α) : ∃ (r : α → α → Prop) [wo : is_well_order α r],
11381137
ord (mk α) = @type α r wo :=

0 commit comments

Comments
 (0)