DEBSOURCES
Skip Quicknav
sources / coq-stdpp / 1.11.0-1 / tests / fin.v
123456
From stdpp Require Import fin. Definition f n m (p : fin n) := m < p. Lemma test : f 47 13 32. Proof. vm_compute. lia. Qed.