File: boolean.v

package info (click to toggle)
mathcomp-zify 1.5.0%2B2.0%2B8.16-4
  • links: PTS, VCS
  • area: main
  • in suites: sid, trixie
  • size: 228 kB
  • sloc: makefile: 43
file content (8 lines) | stat: -rw-r--r-- 209 bytes parent folder | download | duplicates (2)
1
2
3
4
5
6
7
8
From mathcomp Require Import all_ssreflect zify.

Set Implicit Arguments.
Unset Strict Implicit.
Unset Printing Implicit Defensive.

Lemma odd_add (n m : nat) : odd (m + n) = odd m (+) odd n.
Proof. lia. Qed.