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

Commit b07c0f7

Browse files
committed
feat(set_theory/game/basic): Add le_rfl on games (#13814)
1 parent 72816f9 commit b07c0f7

File tree

1 file changed

+4
-2
lines changed

1 file changed

+4
-2
lines changed

src/set_theory/game/basic.lean

Lines changed: 4 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -57,8 +57,10 @@ instance : has_le game :=
5757

5858
-- Adding `@[refl]` and `@[trans]` attributes here would override the ones on
5959
-- `preorder.le_refl` and `preorder.le_trans`, which breaks all non-`game` uses of `≤`!
60-
theorem le_refl : ∀ x : game, x ≤ x :=
61-
by { rintro ⟨x⟩, apply pgame.le_refl }
60+
theorem le_rfl : ∀ {x : game}, x ≤ x :=
61+
by { rintro ⟨x⟩, exact pgame.le_rfl }
62+
theorem le_refl (x : game) : x ≤ x :=
63+
le_rfl
6264
theorem le_trans : ∀ x y z : game, x ≤ y → y ≤ z → x ≤ z :=
6365
by { rintro ⟨x⟩ ⟨y⟩ ⟨z⟩, apply pgame.le_trans }
6466
theorem le_antisymm : ∀ x y : game, x ≤ y → y ≤ x → x = y :=

0 commit comments

Comments
 (0)