|
1 | 1 | (* Distributed under the terms of the MIT license. *) |
2 | 2 | From Coq Require Import Utf8 Program. |
3 | | -From MetaCoq Require Import config utils BasicAst. |
| 3 | +From MetaCoq.Common Require Import config BasicAst. |
| 4 | +From MetaCoq.Utils Require Import utils. |
4 | 5 | From MetaCoq.PCUIC Require PCUICWcbvEval. |
5 | 6 | From MetaCoq.Erasure Require Import EAst EAstUtils ELiftSubst ECSubst EReflect EGlobalEnv |
6 | 7 | EWellformed EWcbvEval. |
| 8 | +From MetaCoq.Utils Require Import bytestring MCString. |
| 9 | +From MetaCoq.Erasure Require Import EWcbvEvalCstrsAsBlocksFixLambdaInd. |
| 10 | +From Coq Require Import BinaryString. |
| 11 | +Import String. |
7 | 12 |
|
8 | 13 | From Equations Require Import Equations. |
9 | 14 | Require Import ssreflect ssrbool. |
@@ -671,10 +676,6 @@ Local Notation "'⊩' v ~ s" := (represents_value v s) (at level 50). |
671 | 676 | Local Hint Constructors represents : core. |
672 | 677 | Local Hint Constructors represents_value : core. |
673 | 678 |
|
674 | | -From MetaCoq Require Import bytestring MCString. |
675 | | -Require Import BinaryString. |
676 | | -Import String. |
677 | | - |
678 | 679 | Fixpoint gen_fresh_aux (na : ident) (Γ : list string) i := |
679 | 680 | match i with |
680 | 681 | | 0 => na |
@@ -1559,8 +1560,6 @@ Proof. |
1559 | 1560 | + eapply All2_All2_Set, All2_app. eapply H1; eauto. econstructor; eauto. |
1560 | 1561 | Qed. |
1561 | 1562 |
|
1562 | | -From MetaCoq Require Import EWcbvEvalCstrsAsBlocksFixLambdaInd. |
1563 | | - |
1564 | 1563 | Lemma lookup_in_env Σ Σ' ind i : |
1565 | 1564 | All2 (fun d d' => d.1 = d'.1 × match d.2 with ConstantDecl (Build_constant_body (Some body)) => |
1566 | 1565 | ∑ body', d'.2 = ConstantDecl (Build_constant_body (Some body')) × [] ;;; [] ⊩ body' ~ body |
|
0 commit comments