Skip to content

Commit

Permalink
Revert "Add some templates (#91)"
Browse files Browse the repository at this point in the history
This reverts commit 0cf0b62.
  • Loading branch information
Ailrun committed Jun 3, 2024
1 parent f8feff0 commit e482c73
Show file tree
Hide file tree
Showing 6 changed files with 2 additions and 68 deletions.
2 changes: 1 addition & 1 deletion theories/Core/Completeness.v
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,7 @@ Import Domain_Notations.

Theorem completeness : forall {Γ M M' A},
{{ Γ ⊢ M ≈ M' : A }} ->
exists W, nbe Γ M A W /\ nbe Γ M' A W.
exists m, nbe Γ M A m /\ nbe Γ M' A m.
Proof with mautosolve.
intros * [env_relΓ]%completeness_fundamental_exp_eq.
destruct_conjs.
Expand Down
12 changes: 0 additions & 12 deletions theories/Core/Semantic/NbE.v
Original file line number Diff line number Diff line change
@@ -1,6 +1,5 @@
From Mcltt Require Import Base LibTactics.
From Mcltt.Core Require Import Evaluation Readback.
From Mcltt.Core Require Export Domain.
Import Domain_Notations.

Generalizable All Variables.
Expand Down Expand Up @@ -61,14 +60,3 @@ Proof.
functional_read_rewrite_clear;
reflexivity.
Qed.

#[export]
Hint Resolve functional_nbe : mcltt.

Ltac functional_nbe_rewrite_clear1 :=
let tactic_error o1 o2 := fail 3 "functional_nbe equality between" o1 "and" o2 "cannot be solved by mauto" in
match goal with
| H1 : nbe ?G ?M ?A ?W, H2 : nbe ?G ?M ?A ?W' |- _ =>
clean replace W' with W by first [solve [mauto] | tactic_error W' W]; clear H2
end.
Ltac functional_nbe_rewrite_clear := repeat functional_nbe_rewrite_clear1.
8 changes: 0 additions & 8 deletions theories/Core/Soundness.v

This file was deleted.

9 changes: 0 additions & 9 deletions theories/Core/Syntactic/Syntax.v
Original file line number Diff line number Diff line change
Expand Up @@ -99,15 +99,6 @@ with ne_to_exp (M : ne) : exp :=
Coercion nf_to_exp : nf >-> exp.
Coercion ne_to_exp : ne >-> exp.

Fact nf_eq_dec : forall (M M' : nf),
({M = M'} + {M <> M'})%type
with ne_eq_dec : forall (M M' : ne),
({M = M'} + {M <> M'})%type.
Proof.
all: intros; decide equality;
apply PeanoNat.Nat.eq_dec.
Defined.

#[global] Declare Custom Entry exp.
#[global] Declare Custom Entry nf.

Expand Down
35 changes: 0 additions & 35 deletions theories/Extraction/TypeCheck.v

This file was deleted.

4 changes: 1 addition & 3 deletions theories/_CoqProject
Original file line number Diff line number Diff line change
Expand Up @@ -37,7 +37,6 @@
./Core/Syntactic/System.v
./Core/Syntactic/System/Definitions.v
./Core/Syntactic/System/Lemmas.v
./Core/Soundness.v
./Core/Soundness/LogicalRelation.v
./Core/Soundness/Weakening.v
./Core/Soundness/Weakening/Definition.v
Expand All @@ -46,7 +45,6 @@
./Frontend/Parser.v
./Frontend/ParserExtraction.v
./Extraction/Evaluation.v
./Extraction/NbE.v
./Extraction/Readback.v
./Extraction/TypeCheck.v
./Extraction/NbE.v
./LibTactics.v

0 comments on commit e482c73

Please sign in to comment.