Zulip Chat Archive

Stream: maths

Topic: Birthday problem


Mario Carneiro (Sep 15 2022 at 07:04):

I see that the birthday problem is listed at https://leanprover-community.github.io/100.html#93 but the theorem statement is a far cry from it:

theorem fintype.card_embedding_eq {α : Type u_1} {β : Type u_2} [fintype α] [fintype β] [fintype (α  β)] :
  fintype.card (α  β) = (fintype.card β).desc_factorial (fintype.card α)

I would expect the full problem to include not just this fact but also the total number of functions from A to B, and then some numerical computation to show that fewer than half of the functions from fin 23 to fin 365 are injective.

Mario Carneiro (Sep 15 2022 at 07:04):

cc: @Eric Rodriguez

Ruben Van de Velde (Sep 15 2022 at 07:06):

That's in archive/100-theorems-list/93_birthday_problem.lean

Kevin Buzzard (Sep 15 2022 at 07:07):

Freek is pretty lenient about what counts :-) Last time I looked, one of the "proofs of Pythagoras' theorem" was a definition of the distance on R2\R^2 for example.

Kevin Buzzard (Sep 15 2022 at 07:08):

But I agree we could do better :-)

Mario Carneiro (Sep 15 2022 at 07:08):

I know that, but that doesn't mean we should be too

Mario Carneiro (Sep 15 2022 at 07:08):

indeed the archive version is much better:

theorem birthday :
  2 * fin 23  fin 365 < fin 23  fin 365  2 * fin 22  fin 365 > fin 22  fin 365

that should be on the web page

Mario Carneiro (Sep 15 2022 at 07:10):

Also a bunch of them have links but no statements on the page, what's up with that?

Alex J. Best (Sep 15 2022 at 08:39):

In a similar vein we have "the Pell equation" but only for d that are one less than a square. It would be a really nice project for someone to solve the full Pell equation sometime

Yaël Dillies (Sep 15 2022 at 08:41):

Wasn't this done on Xena this summer?

Eric Rodriguez (Sep 15 2022 at 08:44):

The archive version was actually a bit more work, as I had to develop the theory of the desc_factorial in order to even get Lean to be able to evaluate the numbers

Eric Rodriguez (Sep 15 2022 at 08:45):

I was hoping to state in terms of probability theory at some point, too, should be relatively easy with the counting measure. I'll update the yaml file when I can sit down at a computer

Kevin Buzzard (Sep 15 2022 at 09:38):

@Harun Khan was working on Pell. I think he got everything: the fundamental unit and a proof that all solutions were up to sign a power of the fundamental unit. Unfortunately he's graduated from Imperial now and is at Stanford doing machine learning :-) I'll see if I can get in touch with him and find out the status of the project.

Kevin Buzzard (Sep 15 2022 at 09:46):

He says it's not public yet but he hopes to make it public within the next couple of weeks

Eric Rodriguez (Sep 16 2022 at 13:30):

Mario Carneiro said:

Also a bunch of them have links but no statements on the page, what's up with that?

I think this is to do with the fact archive is separate, sadly

Mario Carneiro (Sep 16 2022 at 13:34):

Is this file automatically generated? I wouldn't expect it to be

Eric Rodriguez (Sep 16 2022 at 13:34):

I've removed the misleading decl and added some more stuff at #16528

Eric Rodriguez (Sep 16 2022 at 13:34):

Yes, it's generated automatically from 100.yaml

Eric Rodriguez (Sep 16 2022 at 13:39):

I think maybe a manual override to provide some lean code and a link for the cases where it doesn't work would be nice, though

Mario Carneiro (Sep 16 2022 at 13:39):

yeah, I'm thinking to add another key containing markdown to inject in the document

Mario Carneiro (Sep 16 2022 at 13:39):

where's the generator script?

Eric Rodriguez (Sep 16 2022 at 13:56):

they seem to be yaml_check.py/.lean, but they seem a bit small for doing the job they do


Last updated: Dec 20 2023 at 11:08 UTC