Zulip Chat Archive
Stream: mathlib4
Topic: unexpected eliminator resulting type
Maxwell Thum (Jan 14 2023 at 08:39):
In Logic.Encodable.Lattice
,
@[elab_as_elim]
theorem Union_decode₂_cases {f : β → Set α} {C : Set α → Prop} (H0 : C ∅) (H1 : ∀ b, C (f b)) {n} :
C (⋃ b ∈ decode₂ β n, f b)
gives me the error
unexpected eliminator resulting type
C (unionᵢ fun b => unionᵢ fun h => f b)
Maxwell Thum (Jan 14 2023 at 08:40):
Is this an issue with elab_as_elim
? Perhaps a feature?
Eric Wieser (Jan 14 2023 at 08:40):
I think in Lean 3, elab_as_elim
was often just ignored
Maxwell Thum (Jan 14 2023 at 08:41):
Is it safe to just comment it out or delete it then?
Eric Wieser (Jan 14 2023 at 08:41):
Commenting out with a porting note seems fine
Eric Wieser (Jan 14 2023 at 08:42):
But maybe this is a feature that Lean could support
Last updated: Dec 20 2023 at 11:08 UTC