playground/coq/mathcomp/bigop-egs.v

6 lines
148 B
Coq

From mathcomp Require Import all_ssreflect all_algebra.
Lemma sum_odd_3: \sum_(0 <= i < 3.*2 | odd i) i = 3^2.
Proof. by rewrite unlock /=. Qed.