aboutsummaryrefslogtreecommitdiffstats
path: root/src/common/Vericertlib.v
diff options
context:
space:
mode:
authorYann Herklotz <git@yannherklotz.com>2022-09-26 13:13:51 +0100
committerYann Herklotz <git@yannherklotz.com>2022-09-26 13:13:51 +0100
commitd3abe2547c8921d2b324da67370822b7fb89b6c0 (patch)
tree081f017f6c6ce801306d8a7bd70b1c100db88cab /src/common/Vericertlib.v
parent20aae726fa959272ed1568b39b78a0ff501b4882 (diff)
downloadvericert-d3abe2547c8921d2b324da67370822b7fb89b6c0.tar.gz
vericert-d3abe2547c8921d2b324da67370822b7fb89b6c0.zip
Add global monad notation using Instances
This was mostly inspired by the std++ library.
Diffstat (limited to 'src/common/Vericertlib.v')
-rw-r--r--src/common/Vericertlib.v3
1 files changed, 3 insertions, 0 deletions
diff --git a/src/common/Vericertlib.v b/src/common/Vericertlib.v
index 24abece..6f602fc 100644
--- a/src/common/Vericertlib.v
+++ b/src/common/Vericertlib.v
@@ -31,8 +31,11 @@ Require Import compcert.lib.Integers.
Require Import compcert.lib.Maps.
Require Import vericert.common.Show.
+Require Export vericert.common.Monad.
Require Export vericert.common.Optionmonad.
+#[global] Open Scope vericert_scope.
+
(* Depend on CompCert for the basic library, as they declare and prove some
useful theorems. *)