Zulip Chat Archive

Stream: lean4

Topic: Idiomatic unit test


Geoffrey Irving (Jan 06 2024 at 20:25):

If I have a computational expression expr : Bool, and want to record a unit test that expr = True, I can do

lemma test : expr := by native_decide

Is this the most idiomatic way to express a unit test, or there is something better?

Henrik Böving (Jan 06 2024 at 20:33):

See https://leanprover.zulipchat.com/#narrow/stream/270676-lean4/topic/How.20to.20unit.2Fdoc.20test.3F


Last updated: May 02 2025 at 03:31 UTC