From fdf9a8a09f73c531aa7fc0e96cad02dd6011e2c9 Mon Sep 17 00:00:00 2001 From: Jacques-Henri Jourdan Date: Mon, 4 May 2020 11:37:49 +0200 Subject: Coq-MenhirLib: explicit import ListNotations (#354) import ListNotations wherever it is necessary so that we do not rely on it being exported by Program. (See #352.) This is a backport from upstream: https://gitlab.inria.fr/fpottier/menhir/-/commit/53f94fa42c80ab1728383e9d2b19006180b14a78 --- MenhirLib/Interpreter.v | 2 ++ 1 file changed, 2 insertions(+) (limited to 'MenhirLib/Interpreter.v') diff --git a/MenhirLib/Interpreter.v b/MenhirLib/Interpreter.v index 568597ba..c36ca614 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. @@ -82,6 +83,7 @@ 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. -- cgit