Skip to content

Commit

Permalink
clean up
Browse files Browse the repository at this point in the history
  • Loading branch information
kik committed Jul 25, 2010
1 parent b92c8e0 commit b83681d
Show file tree
Hide file tree
Showing 3 changed files with 517 additions and 676 deletions.
13 changes: 12 additions & 1 deletion coq/tarai/Denotation.v
Original file line number Diff line number Diff line change
Expand Up @@ -223,6 +223,17 @@ Proof.
exact H.
Qed.

Theorem ntarai_continuous_v: forall n v v' x, le v v' ->
ntarai n v = V x -> ntarai n v' = V x.
Proof.
intros.
generalize (ntarai_continuous n v v' H).
rewrite H0.
intro.
inversion H1.
auto.
Qed.

Lemma Y_add: forall A n m (init: A) (recur: A -> A),
Yn (n+m)%nat init recur = Yn n (Yn m init recur) recur.
Proof.
Expand All @@ -236,7 +247,7 @@ Qed.
Definition f_le `{aord: PreOrder a, bord: PreOrder b} (f g: a -> b) :=
forall v, le (f v) (g v).

Instance CFOrder `{aord: PreOrder a, bord: PreOrder b} : PreOrder (a -> b) := {
Instance FOrder `{aord: PreOrder a, bord: PreOrder b} : PreOrder (a -> b) := {
le := f_le
}.
Proof.
Expand Down
Loading

0 comments on commit b83681d

Please sign in to comment.