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

Commit be79f9f

Browse files
gebnerdigama0
authored andcommitted
chore(data/cardinal): put embedding into cardinal namespace
1 parent ee7ede9 commit be79f9f

File tree

2 files changed

+6
-2
lines changed

2 files changed

+6
-2
lines changed

data/cardinal.lean

Lines changed: 5 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -20,6 +20,8 @@ local attribute [instance] prop_decidable
2020

2121
universes u v w x
2222

23+
namespace cardinal
24+
2325
structure embedding (α : Sort*) (β : Sort*) :=
2426
(to_fun : α → β)
2527
(inj : injective to_fun)
@@ -224,7 +226,9 @@ let f' : (α → γ) → (β → γ) := λf b, if h : ∃c, e c = b then f (some
224226

225227
end embedding
226228

227-
protected def equiv.to_embedding {α : Type u} {β : Type v} (f : α ≃ β) : embedding α β :=
229+
end cardinal
230+
231+
protected def equiv.to_embedding {α : Type u} {β : Type v} (f : α ≃ β) : cardinal.embedding α β :=
228232
⟨f, f.bijective.1
229233

230234
@[simp] theorem equiv.to_embedding_coe_fn {α : Type u} {β : Type v} (f : α ≃ β) :

data/ordinal.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -10,7 +10,7 @@ Ordinals are defined as equivalences of well-ordered sets by order isomorphism.
1010
import data.cardinal
1111
noncomputable theory
1212

13-
open function
13+
open function cardinal
1414
local attribute [instance] classical.prop_decidable
1515

1616
universes u v w

0 commit comments

Comments
 (0)