Skip to content

Commit

Permalink
doc(set_theory/game/basic): improve docs (#14268)
Browse files Browse the repository at this point in the history
  • Loading branch information
vihdzp committed May 22, 2022
1 parent cef5898 commit 5a24374
Showing 1 changed file with 6 additions and 5 deletions.
11 changes: 6 additions & 5 deletions src/set_theory/game/basic.lean
Expand Up @@ -9,15 +9,16 @@ import tactic.abel
/-!
# Combinatorial games.
In this file we define the quotient of pre-games by the equivalence relation `p ≈ q ↔ p ≤ q ∧ q ≤
p`, and construct an instance `add_comm_group game`, as well as an instance `partial_order game`.
In this file we define the quotient of pre-games by the equivalence relation
`p ≈ q ↔ p ≤ q ∧ q ≤ p` (its `antisymmetrization`), and construct an instance `add_comm_group game`,
as well as an instance `partial_order game`.
## Multiplication on pre-games
We define the operations of multiplication and inverse on pre-games, and prove a few basic theorems
about them. Multiplication is not well-behaved under equivalence of pre-games i.e. `x.equiv y` does
not imply `(x*z).equiv (y*z)`. Hence, multiplication is not a well-defined operation on games.
Nevertheless, the abelian group structure on games allows us to simplify many proofs for pre-games.
about them. Multiplication is not well-behaved under equivalence of pre-games i.e. `xy` does not
imply `x * z ≈ y * z`. Hence, multiplication is not a well-defined operation on games. Nevertheless,
the abelian group structure on games allows us to simplify many proofs for pre-games.
-/

open function
Expand Down

0 comments on commit 5a24374

Please sign in to comment.