DEBSOURCES
Skip Quicknav
sources / coq / 8.20.1%2Bdfsg-1 / test-suite / bugs / bug_5145.v
12345678910
Class instructions := { W : Type; ldi : nat -> W }. Fail Definition foo := let y2 := ldi 0 in let '(CF, _) := (true, 0) in y2.