File: test_5_3.v

package info (click to toggle)
coq-hierarchy-builder 1.8.1-1
  • links: PTS, VCS
  • area: main
  • in suites: forky, sid, trixie
  • size: 1,988 kB
  • sloc: makefile: 109
file content (20 lines) | stat: -rw-r--r-- 524 bytes parent folder | download | duplicates (2)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
From Coq Require Import ZArith ssreflect.
From HB Require Import structures.
From HB Require Import demo1.hierarchy_5.

HB.instance
Definition Z_AddComoid := AddComoid_of_TYPE.Build
  Z 0%Z Z.add
  Z.add_assoc Z.add_comm Z.add_0_l.

HB.instance
Definition Z_SemiRing := SemiRing_of_AddComoid.Build
  Z 1%Z Z.mul
  Z.mul_assoc Z.mul_1_l Z.mul_1_r
  Z.mul_add_distr_r Z.mul_add_distr_l
  Z.mul_0_l Z.mul_0_r.

Open Scope hb_scope.

Example test1 (m n : Z) : m + n * 0 * 0 = m.
Proof. by rewrite -mulrA !mulr0 addrC add0r. Qed.