aboutsummaryrefslogtreecommitdiffstats
path: root/src/common/Coquplib.v
diff options
context:
space:
mode:
authorJames Pollard <james@pollard.dev>2020-06-28 15:06:17 +0100
committerJames Pollard <james@pollard.dev>2020-06-28 15:06:17 +0100
commit8fda19cb580bda72f374bc2176d7e2efa5cd613b (patch)
tree5d41327ab5c692ed2bc2319a9568d2ff596cd2dd /src/common/Coquplib.v
parentbb80bc5d196665498f7b365e9e26468ed5999ea9 (diff)
downloadvericert-8fda19cb580bda72f374bc2176d7e2efa5cd613b.tar.gz
vericert-8fda19cb580bda72f374bc2176d7e2efa5cd613b.zip
Work on proof.
Diffstat (limited to 'src/common/Coquplib.v')
-rw-r--r--src/common/Coquplib.v3
1 files changed, 3 insertions, 0 deletions
diff --git a/src/common/Coquplib.v b/src/common/Coquplib.v
index b4ca906..b8a02d2 100644
--- a/src/common/Coquplib.v
+++ b/src/common/Coquplib.v
@@ -117,6 +117,9 @@ Ltac simplify := unfold_constants; simpl in *;
Global Opaque Nat.div.
Global Opaque Z.mul.
+Infix "==nat" := eq_nat_dec (no associativity, at level 50).
+Infix "==Z" := Z.eq_dec (no associativity, at level 50).
+
(* Definition const (A B : Type) (a : A) (b : B) : A := a.
Definition compose (A B C : Type) (f : B -> C) (g : A -> B) (x : A) : C := f (g x). *)