Zulip Chat Archive

Stream: new members

Topic: computing satisfying instance?


Mark Aagaard (Oct 11 2024 at 21:40):

Is there an existing mechanism to compute a satisfying instance of a propositional formula? For example (pq)¬r(p \vee q) \wedge \neg r would return p¬rp \wedge \neg r.

-mark

Daniel Weber (Oct 12 2024 at 10:34):

What do you need it for?

import Mathlib.Tactic

example {p q r : Bool} (h : (p  q)  ¬ r) : False := by
  slim_check

can give you an example assignment

Mark Aagaard (Oct 12 2024 at 22:57):

Thanks, Daniel. This is great.

I'm teaching an intro to logic and verification course and want to show off some of the features of Lean4 as it relates to exercises that the students have done by hand.

-mark


Last updated: May 02 2025 at 03:31 UTC