aboutsummaryrefslogtreecommitdiffstats
path: root/MenhirLib/Interpreter.v
diff options
context:
space:
mode:
Diffstat (limited to 'MenhirLib/Interpreter.v')
-rw-r--r--MenhirLib/Interpreter.v1
1 files changed, 1 insertions, 0 deletions
diff --git a/MenhirLib/Interpreter.v b/MenhirLib/Interpreter.v
index 568597ba..07aeae5a 100644
--- a/MenhirLib/Interpreter.v
+++ b/MenhirLib/Interpreter.v
@@ -12,6 +12,7 @@
(****************************************************************************)
From Coq Require Import List Syntax.
+Import ListNotations.
From Coq.ssr Require Import ssreflect.
Require Automaton.
Require Import Alphabet Grammar Validator_safe.