aboutsummaryrefslogtreecommitdiffstats
path: root/src/array/Array_checker.v
diff options
context:
space:
mode:
authorckeller <ckeller@users.noreply.github.com>2019-03-11 20:25:35 +0100
committerGitHub <noreply@github.com>2019-03-11 20:25:35 +0100
commita88e3b3b6ad01a9b85c828b9a1225732275affee (patch)
treeacc3768695698a80867b4ce941ab4cb7b4b99d7a /src/array/Array_checker.v
parent33010bfa6345549d8b9b0c06f44150b60d0c86e5 (diff)
downloadsmtcoq-a88e3b3b6ad01a9b85c828b9a1225732275affee.tar.gz
smtcoq-a88e3b3b6ad01a9b85c828b9a1225732275affee.zip
V8.8 (#42)
* Towards 8.8 * Towards 8.8 * Towards 8.8 * Towards 8.8 * Towards 8.8 * Towards 8.8 * Towards 8.8 * Organization structures * 8.8 ok with standard coq
Diffstat (limited to 'src/array/Array_checker.v')
-rw-r--r--src/array/Array_checker.v6
1 files changed, 2 insertions, 4 deletions
diff --git a/src/array/Array_checker.v b/src/array/Array_checker.v
index dd1a65f..3a982b2 100644
--- a/src/array/Array_checker.v
+++ b/src/array/Array_checker.v
@@ -10,8 +10,8 @@
(**************************************************************************)
-Require Import Bool List Int63 PArray SMT_classes.
-Require Import Misc State SMT_terms FArray.
+Require Import Bool List Int63 PArray Psatz.
+Require Import Misc State SMT_terms FArray SMT_classes.
Import Form.
Import Atom.
@@ -897,8 +897,6 @@ Section certif.
afold_left bool int false orb (Lit.interp rho) a =
C.interp rho (to_list a).
- Require Import Psatz.
-
Lemma valid_check_ext lres : C.valid rho (check_ext lres).
unfold check_ext, eq_sel_sym.
case_eq (Lit.is_pos lres); intro Heq; simpl; try now apply C.interp_true.