Zulip Chat Archive

Stream: lean4

Topic: injection error


Nick Chopper (Jan 30 2021 at 10:06):

theorem subtype_inj (A: Type) (p: A  Prop) (a b: A) (pa: p a) (pb: p b) : (⟨a, pa⟩: {a//p a}) = (⟨b, pb⟩: {b//p b})  a = b := by
  intro eq
  injection eq
  assumption

results in (red line at injection eq)

tactic 'introN' failed, insufficient number of binders
A : Type
p : A  Prop
a b : A
pa : p a
pb : p b
 : a = b
 a = b

Leonardo de Moura (Jan 30 2021 at 20:01):

Pushed a fix https://github.com/leanprover/lean4/commit/b7a0bdb9c9ba6adade3650c560435031b5cdfa99


Last updated: Dec 20 2023 at 11:08 UTC