lean2/tests/lean/run/cast_sorry_bug.lean

12 lines
383 B
Text
Raw Normal View History

import logic data.nat
open nat
inductive fin : → Type :=
| zero : Π {n : }, fin (succ n)
| succ : Π {n : }, fin n → fin (succ n)
theorem foo (n m : ) (a : fin n) (b : fin m) (H : n = m) : cast (congr_arg fin H) a = b :=
have eq : fin n = fin m, from congr_arg fin H,
have ceq : cast eq a = b, from sorry, -- sorry implicit argument must have access to eq
sorry