Zulip Chat Archive

Stream: general

Topic: Metis Theorem Prover in Lean


A. Stone Olguin (Jun 10 2021 at 20:03):

Hi all, I was wondering if anyone knows if anyone has worked on implementing the metis theorem prover in Lean similar to how it was implemented in Isabelle. Any info helps, thanks!

Gabriel Ebner (Jun 10 2021 at 20:11):

Some time back I wrote a superposition in Lean, which fills a similar niche as metis. https://github.com/leanprover/super
Lean 3 was quite slow though, making this tool less useful than it could be. Lean 4 is out now, so at some point I am going to revisit super and see if I can make it faster this time.

Max (Jun 12 2021 at 21:09):

On a related note, is there any ongoing projects at a Sledgehammer for Lean4?

Patrick Massot (Jun 12 2021 at 21:19):

There are a lot of people who are at least thinking really seriously about whether this is the right question to ask.

Patrick Massot (Jun 12 2021 at 21:19):

see https://matryoshka-project.github.io/ in particular

Brandon Brown (Jun 13 2021 at 03:24):

Isnt Lean-GPTF basically developing into a sledgehammer?

Alexander Bentkamp (Jun 13 2021 at 06:55):

Brandon Brown: Isnt Lean-GPTF basically developing into a sledgehammer?

In the sense that both offer general purpose automation, yes, but the technology behind the scenes is very different. GPTF relies on neural networks, whereas sledgehammer calls first-order automated theorem provers, such as Vampire or E.

Max (Jun 13 2021 at 13:11):

Nice, gonna read through those sources! Thanks :)


Last updated: Dec 20 2023 at 11:08 UTC