aboutsummaryrefslogtreecommitdiffstats
path: root/src/Misc.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/Misc.v')
-rw-r--r--src/Misc.v9
1 files changed, 8 insertions, 1 deletions
diff --git a/src/Misc.v b/src/Misc.v
index fe724f4..84feab4 100644
--- a/src/Misc.v
+++ b/src/Misc.v
@@ -10,7 +10,7 @@
(**************************************************************************)
-Require Import Bool List PArray Int63.
+Require Import Bool List PArray Int63 ZArith.
Local Open Scope int63_scope.
Local Open Scope array_scope.
@@ -1038,3 +1038,10 @@ Proof. destruct b; intuition. Qed.
Lemma is_true_iff e : e = true <-> is_true e.
Proof. now unfold is_true. Qed.
+
+
+(*
+ Local Variables:
+ coq-load-path: ((rec "." "SMTCoq"))
+ End:
+*)