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

Commit

Permalink
feat(set_theory/ordinal_arithmetic): Proved add_log_le_log_mul (#11228
Browse files Browse the repository at this point in the history
)

That is, `log b u + log b v ≤ log b (u * v)`. The other direction holds only when `b ≠ 2` and `b` is principal multiplicative, and will be added at a much later PR.
  • Loading branch information
vihdzp committed Jan 4, 2022
1 parent 18330f6 commit 5f3f01f
Showing 1 changed file with 9 additions and 0 deletions.
9 changes: 9 additions & 0 deletions src/set_theory/ordinal_arithmetic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -1208,6 +1208,15 @@ if b1 : 1 < b then
le_trans (le_power_self _ b1) (power_log_le b (ordinal.pos_iff_ne_zero.2 x0))
else by simp only [log_not_one_lt b1, ordinal.zero_le]

theorem add_log_le_log_mul {x y : ordinal} (b : ordinal) (x0 : 0 < x) (y0 : 0 < y) :
log b x + log b y ≤ log b (x * y) :=
begin
by_cases hb : 1 < b,
{ rw [le_log hb (mul_pos x0 y0), power_add],
exact mul_le_mul (power_log_le b x0) (power_log_le b y0) },
simp only [log_not_one_lt hb, zero_add]
end

/-! ### The Cantor normal form -/

theorem CNF_aux {b o : ordinal} (b0 : b ≠ 0) (o0 : o ≠ 0) :
Expand Down

0 comments on commit 5f3f01f

Please sign in to comment.