Zulip Chat Archive

Stream: lean4

Topic: Nontransitivity of DefEq


Chris Hughes (Jan 23 2023 at 14:02):

I came across this nontransitivity of DefEq today that isn't anything to do with Prop or Quotients. rfl cannot prove the following lemma.

example {α : Type} (f g : α  Unit) : f = g :=
  calc f
    = fun x => f x := rfl
  _ = g := rfl

Reid Barton (Jan 23 2023 at 14:03):

This is supposed to be by eta for functions + eta for Unit?

Chris Hughes (Jan 23 2023 at 14:04):

Yes


Last updated: Dec 20 2023 at 11:08 UTC