From 3bd82b3cb10a721f2e2c8db6d0271c83a22095a3 Mon Sep 17 00:00:00 2001 From: Xavier Leroy Date: Mon, 13 Feb 2017 11:15:34 +0100 Subject: Use "Local" as prefix Open Local becomes Local Open. This silences Coq 8.6's warning. Also: remove one useless Require-inside-a-module that caused another warning. --- backend/SelectDiv.vp | 2 +- 1 file changed, 1 insertion(+), 1 deletion(-) (limited to 'backend/SelectDiv.vp') diff --git a/backend/SelectDiv.vp b/backend/SelectDiv.vp index 5cc66322..dc85fb25 100644 --- a/backend/SelectDiv.vp +++ b/backend/SelectDiv.vp @@ -17,7 +17,7 @@ Require Import Compopts. Require Import AST Integers Floats. Require Import Op CminorSel SelectOp SplitLong SelectLong. -Open Local Scope cminorsel_scope. +Local Open Scope cminorsel_scope. (** We try to turn divisions by a constant into a multiplication by a pseudo-inverse of the divisor. The approach is described in -- cgit