From a88e3b3b6ad01a9b85c828b9a1225732275affee Mon Sep 17 00:00:00 2001 From: ckeller Date: Mon, 11 Mar 2019 20:25:35 +0100 Subject: 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 --- src/array/Array_checker.v | 6 ++---- 1 file changed, 2 insertions(+), 4 deletions(-) (limited to 'src/array/Array_checker.v') 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. -- cgit