aboutsummaryrefslogtreecommitdiff
path: root/src/Util/ZUtil/Mul.v
blob: 6cf851e4e6378d92a2e68fe22c874ca7adb75d53 (plain)
1
2
3
4
5
6
7
8
Require Import Coq.ZArith.ZArith.
Require Import Coq.micromega.Lia.
Local Open Scope Z_scope.

Module Z.
  Lemma mul_comm3 x y z : x * (y * z) = y * (x * z).
  Proof. lia. Qed.
End Z.