aboutsummaryrefslogtreecommitdiffstats
path: root/src/array/FArray.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/FArray.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/FArray.v')
-rw-r--r--src/array/FArray.v5
1 files changed, 2 insertions, 3 deletions
diff --git a/src/array/FArray.v b/src/array/FArray.v
index 1f8c6b4..a17817f 100644
--- a/src/array/FArray.v
+++ b/src/array/FArray.v
@@ -11,7 +11,8 @@
Require Import Bool OrderedType SMT_classes.
-Require Import ProofIrrelevance. (* TODO: REMOVE THIS AXIOM *)
+Require Import ProofIrrelevance Classical_Pred_Type ClassicalEpsilon. (* TODO: REMOVE ALL THESE AXIOMS *)
+
(** This file formalizes functional arrays with extensionality as specified in
SMT-LIB 2. It gives realization to axioms that define the SMT-LIB theory of
@@ -1777,8 +1778,6 @@ Section FArray.
Section Classical_extensionnality.
- Require Import Classical_Pred_Type ClassicalEpsilon.
-
Lemma extensionnality2 : forall a b, a <> b -> (exists i, select a i <> select b i).
Proof.
intros.