leanprover-community / mathlib

  • Home
  • Zulip archive
  • API documentation
  • Lean web editor
  • Links

Zulip Chat Archive

Stream: lean4

Topic: thunk simp


awalterschulze (Nov 11 2022 at 08:26):

How does one cases on a Thunk in a proof?

def f (c : Thunk Bool) (x : Nat) : Nat :=
  if c.get then
    x
  else
    0

theorem f1 (b: Thunk Bool): f b 0 = 0 := by

Sebastian Ullrich (Nov 11 2022 at 08:31):

Unfold f and case on b.get


Last updated: May 02 2025 at 03:31 UTC

Theme Simple by wildflame © 2016 Powered by jekyll