Skip to content

Commit

Permalink
Refactor context file to use sigma library
Browse files Browse the repository at this point in the history
  • Loading branch information
takanuva committed Oct 2, 2024
1 parent 3e6933e commit 1b202e3
Show file tree
Hide file tree
Showing 2 changed files with 22 additions and 0 deletions.
1 change: 1 addition & 0 deletions theories/Context.v
Original file line number Diff line number Diff line change
Expand Up @@ -8,6 +8,7 @@ Require Export Setoid.
Require Export Relations.
Require Import Equality.
Require Import Local.Prelude.
Require Import Local.Substitution.
Require Import Local.Syntax.
Require Import Local.Metatheory.

Expand Down
21 changes: 21 additions & 0 deletions theories/Metatheory.v
Original file line number Diff line number Diff line change
Expand Up @@ -1251,3 +1251,24 @@ Proof with modulo_arith.
rewrite Nat.add_comm.
assumption.
Qed.

Lemma apply_parameters_unfold:
forall y ys k e,
apply_parameters (y :: ys) k e = subst y k (apply_parameters ys (1 + k) e).
Proof.
intros.
unfold apply_parameters.
now sigma.
Qed.

Lemma right_cycle_characterization:
forall i k e,
right_cycle i k e =
apply_parameters (high_sequence i ++ [bound 0]) k (lift (S i) (S i + k) e).
Proof.
intros.
unfold right_cycle.
unfold apply_parameters.
assert (length (high_sequence i) = i) by apply sequence_length.
now sigma.
Qed.

0 comments on commit 1b202e3

Please sign in to comment.