Open LukasMias opened 1 year ago
I'm not sure whether casesm _
is supposed to work or not, but at least there's a workaround here, if you know the name of the type:
theorem mwe : ∀ (x : twoPoints), x = zero ∨ x = one := fun x ↦ by cases_type twoPoints <;> simp
In lean 3:
In lean 4:
Not sure if this was intended behavior, but it was definitely used in mathlib3, e.g. data.sign, so some proofs break now. Related Zulip thread: here.