Zulip Chat Archive

Stream: general

Topic: Simplifying nested lambda expressions


Ken Roe (Jan 12 2019 at 00:15):

It appears that "simp" is not completely robust. How do I get the following simplification to work?

theorem beta_r {y:  } : (λ (q:) (z:), y z)=(λ (r:), y) :=
begin
    simp
end

Bryan Gin-ge Chen (Jan 12 2019 at 00:21):

The simp seems to work for me. What version of lean are you using / what else do you have in the file?

Bryan Gin-ge Chen (Jan 12 2019 at 00:23):

The squeeze_simp tactic in mathlib's tactic.squeeze tells me that simp only [eq_self_iff_true] ought to work too.

Ken Roe (Jan 12 2019 at 00:32):

I'm using Lean 3.4.1. Should I update?

Ken Roe (Jan 12 2019 at 00:34):

It does work--I realized I need to type a "," after the "simp" to see the reduction show up in the editor.


Last updated: Dec 20 2023 at 11:08 UTC