DEBSOURCES
Skip Quicknav
sources / coq-hierarchy-builder / 1.8.1-1 / tests / fix_loop.v
1234
From HB Require Import structures. HB.mixin Record M A := { x: nat }. HB.structure Definition S := { A of M A }.