Birthday Problem #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
This file proves Theorem 93 from the 100 Theorems List.
As opposed to the standard probabilistic statement, we instead state the birthday problem
in terms of injective functions. The general result about fintype.card (α ↪ β)
which this proof
uses is fintype.card_embedding_eq
.
Birthday Problem: set cardinality interpretation.
@[protected, instance]
Equations
@[protected, instance]
@[protected, instance]
noncomputable
def
theorems_100.pi.measure_theory.measure_space
{n m : ℕ} :
measure_theory.measure_space (fin n → fin m)
theorem
theorems_100.birthday_measure
:
⇑measure_theory.measure_space.volume {f : fin 23 → fin 365 | function.injective f} < 1 / 2
Birthday Problem: first probabilistic interpretation.