diff options
| -rw-r--r-- | theories/Bool/Bvector.v | 3 | ||||
| -rwxr-xr-x | theories/Bool/Zerob.v | 3 | ||||
| -rw-r--r-- | theories/ZArith/zarith_aux.v | 3 |
3 files changed, 9 insertions, 0 deletions
diff --git a/theories/Bool/Bvector.v b/theories/Bool/Bvector.v index f26a83f837..c874ecd11c 100644 --- a/theories/Bool/Bvector.v +++ b/theories/Bool/Bvector.v @@ -14,6 +14,9 @@ Require Export Bool. Require Export Sumbool. Require Arith. +V7only [Import nat_scope.]. +Open Local Scope nat_scope. + (* On s'inspire de PolyList pour fabriquer les vecteurs de bits. La dimension du vecteur est un paramètre trop important pour diff --git a/theories/Bool/Zerob.v b/theories/Bool/Zerob.v index 07b4c68c8e..7880251619 100755 --- a/theories/Bool/Zerob.v +++ b/theories/Bool/Zerob.v @@ -11,6 +11,9 @@ Require Arith. Require Bool. +V7only [Import nat_scope.]. +Open Local Scope nat_scope. + Definition zerob : nat->bool := [n:nat]Cases n of O => true | (S _) => false end. diff --git a/theories/ZArith/zarith_aux.v b/theories/ZArith/zarith_aux.v index fc0abca952..936468fef7 100644 --- a/theories/ZArith/zarith_aux.v +++ b/theories/ZArith/zarith_aux.v @@ -12,6 +12,9 @@ Require Arith. Require Export fast_integer. +V7only [Import nat_scope.]. +Open Local Scope nat_scope. + Tactic Definition ElimCompare com1 com2:= Elim (Dcompare (Zcompare com1 com2)); [ Idtac |
