DEBSOURCES
Skip Quicknav
sources / coq-doc / 8.20.0-2 / test-suite / bugs / bug_5617.v
12345678
Set Primitive Projections. Record T X := { F : X }. Fixpoint f (n : nat) : nat := match n with | 0 => 0 | S m => F _ {| F := f |} m end.