aboutsummaryrefslogtreecommitdiffstats
path: root/scheduling/RTLpath.v
diff options
context:
space:
mode:
Diffstat (limited to 'scheduling/RTLpath.v')
-rw-r--r--scheduling/RTLpath.v2
1 files changed, 0 insertions, 2 deletions
diff --git a/scheduling/RTLpath.v b/scheduling/RTLpath.v
index 0f303597..a4fce97e 100644
--- a/scheduling/RTLpath.v
+++ b/scheduling/RTLpath.v
@@ -28,8 +28,6 @@ Require Import Op Registers.
Require Import RTL Linking.
Require Import Lia.
-Declare Scope option_monad_scope.
-
Notation "'SOME' X <- A 'IN' B" := (match A with Some X => B | None => None end)
(at level 200, X ident, A at level 100, B at level 200)
: option_monad_scope.