CoqDSC.LambdaAL
Base terms
Grammar for base terms
- "Var x" represents "\(x\)".
- "Def f x t" represents "\({\bf let }\; y = f\, x \;{\bf in }\; t\)".
- "DefTuple [x₁; ...; xₙ]" represents "\({\bf let }\; y = (x₁, ..., xₙ) \;{\bf in }\; t\)".
Inductive term :=
| Var : var -> term
| Def : var -> var -> term -> term
| DefTuple : list var -> term -> term.
| Var : var -> term
| Def : var -> var -> term -> term
| DefTuple : list var -> term -> term.
Syntactic sugar
Definition call f x := Def f x (Var (Idx O)).
Notation "@( f , x )" := (call f x).
Definition ttuple xs := DefTuple xs (Var (Idx 0)).
Notation "@( f , x )" := (call f x).
Definition ttuple xs := DefTuple xs (Var (Idx 0)).
The type of change terms. (Figure 1 in paper.)
Notice that we could have used the same syntax as term to
represent change terms since they are totally isomorphic. Yet, we
prefer a form of "strong" typing in the formalization to avoid any
confusion in the definitions, in particular in the operational
semantics, in the program transformation and the validity
relation.
- "dVar x" represents "\(dx\)".
- "dDef f x dt" represents "\({\bf let}\; y = f\, x, dy = df\, x\, dx\, {\bf in}\, dt\)".
- "dDefTuple [dx₁; ...; dxₙ] dt" represents "\({\bf let}\; y = (x₁, ..., xₙ), dy = (dx₁, ..., dxₙ) \, {\bf in}\, dt\)".
Inductive dterm :=
| dVar : dvar -> dterm
| dDef : var -> var -> dterm -> dterm
| dDefTuple : list dvar -> dterm -> dterm.
Definition dcall f x := dDef f x (dVar (d (Idx O))).
Definition dttuple xs := dDefTuple xs (dVar (d (Idx 0))).
| dVar : dvar -> dterm
| dDef : var -> var -> dterm -> dterm
| dDefTuple : list dvar -> dterm -> dterm.
Definition dcall f x := dDef f x (dVar (d (Idx O))).
Definition dttuple xs := dDefTuple xs (dVar (d (Idx 0))).
Definition und (dx : dvar) : var :=
match dx with d x => x end.
Lemma d_und:
forall dx, d (und dx) = dx.
Proof. destruct dx. auto. Qed.
Lemma und_d:
forall x, und (d x) = x.
Proof. destruct x. auto. Qed.
Lemma map_und_d_id :
forall xs, List.map und (List.map d xs) = xs.
Proof.
induction xs; simpl; eauto.
rewrite IHxs. auto.
Qed.
Definition context := term.
Fixpoint graft (ctx : context) (u : term) : term :=
match ctx with
| Var _ => u
| DefTuple xs ctx => DefTuple xs (graft ctx u)
| Def f x ctx => Def f x (graft ctx u)
end.
Definition dcontext := dterm.
Fixpoint dgraft (dctx : dcontext) (du : dterm) : dterm :=
match dctx with
| dVar _ => du
| dDefTuple xs dctx => dDefTuple xs (dgraft dctx du)
| dDef f x dctx => dDef f x (dgraft dctx du)
end.
match dx with d x => x end.
Lemma d_und:
forall dx, d (und dx) = dx.
Proof. destruct dx. auto. Qed.
Lemma und_d:
forall x, und (d x) = x.
Proof. destruct x. auto. Qed.
Lemma map_und_d_id :
forall xs, List.map und (List.map d xs) = xs.
Proof.
induction xs; simpl; eauto.
rewrite IHxs. auto.
Qed.
Definition context := term.
Fixpoint graft (ctx : context) (u : term) : term :=
match ctx with
| Var _ => u
| DefTuple xs ctx => DefTuple xs (graft ctx u)
| Def f x ctx => Def f x (graft ctx u)
end.
Definition dcontext := dterm.
Fixpoint dgraft (dctx : dcontext) (du : dterm) : dterm :=
match dctx with
| dVar _ => du
| dDefTuple xs dctx => dDefTuple xs (dgraft dctx du)
| dDef f x dctx => dDef f x (dgraft dctx du)
end.