diff options
| author | letouzey | 2012-07-05 16:56:28 +0000 |
|---|---|---|
| committer | letouzey | 2012-07-05 16:56:28 +0000 |
| commit | a46ccd71539257bb55dcddd9ae8510856a5c9a16 (patch) | |
| tree | f5934c98bd6288cc485f20dd9dfeae598170697e /plugins | |
| parent | 8e33b709fb2225d256dccfd4b071f85144d92d45 (diff) | |
Open Local Scope ---> Local Open Scope, same with Notation and alii
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@15517 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'plugins')
| -rw-r--r-- | plugins/omega/PreOmega.v | 2 | ||||
| -rw-r--r-- | plugins/ring/LegacyArithRing.v | 2 | ||||
| -rw-r--r-- | plugins/setoid_ring/RealField.v | 2 |
3 files changed, 3 insertions, 3 deletions
diff --git a/plugins/omega/PreOmega.v b/plugins/omega/PreOmega.v index bc08deaf9c..cc6a7066a9 100644 --- a/plugins/omega/PreOmega.v +++ b/plugins/omega/PreOmega.v @@ -8,7 +8,7 @@ Require Import Arith Max Min BinInt BinNat Znat Nnat. -Open Local Scope Z_scope. +Local Open Scope Z_scope. (** * zify: the Z-ification tactic *) diff --git a/plugins/ring/LegacyArithRing.v b/plugins/ring/LegacyArithRing.v index fd5bcd9355..94dc48a733 100644 --- a/plugins/ring/LegacyArithRing.v +++ b/plugins/ring/LegacyArithRing.v @@ -13,7 +13,7 @@ Require Export LegacyRing. Require Export Arith. Require Import Eqdep_dec. -Open Local Scope nat_scope. +Local Open Scope nat_scope. Fixpoint nateq (n m:nat) {struct m} : bool := match n, m with diff --git a/plugins/setoid_ring/RealField.v b/plugins/setoid_ring/RealField.v index 14c4270f9a..1cbddc27de 100644 --- a/plugins/setoid_ring/RealField.v +++ b/plugins/setoid_ring/RealField.v @@ -5,7 +5,7 @@ Require Import Rdefinitions. Require Import Rpow_def. Require Import Raxioms. -Open Local Scope R_scope. +Local Open Scope R_scope. Lemma RTheory : ring_theory 0 1 Rplus Rmult Rminus Ropp (eq (A:=R)). Proof. |
