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, 0 insertions, 1 deletions
diff --git a/MenhirLib/Interpreter.v b/MenhirLib/Interpreter.v
index c36ca614..07aeae5a 100644
--- a/MenhirLib/Interpreter.v
+++ b/MenhirLib/Interpreter.v
@@ -83,7 +83,6 @@ Proof. by rewrite /cast -Eqdep_dec.eq_rect_eq_dec. Qed.
CoInductive buffer : Type :=
Buf_cons { buf_head : token; buf_tail : buffer }.
-Declare Scope buffer_scope.
Delimit Scope buffer_scope with buf.
Bind Scope buffer_scope with buffer.