我试图在Coq中形式化简单类型的lambda演算并且有一个问题,说明在空上下文中良好类型表达式的自由变量集是空的。
以下是可能形式化的相关部分。
Require Import Coq.Arith.Arith.
Require Import Coq.MSets.MSets.
Require Import Coq.FSets.FMaps.
Inductive type : Set :=
| tunit : type
| tfun : type -> type -> type.
Module Var := Nat.
Definition var : Set := Var.t.
Module VarSet := MSetAVL.Make Var.
Module VarSetFacts := MSetFacts.Facts VarSet.
Module VarSetProps := MSetProperties.Properties VarSet.
Module Context := FMapWeakList.Make Var.
Module ContextFacts := FMapFacts.Facts Context.
Module ContextProps := FMapFacts.Properties Context.
Definition context := Context.t type.
Definition context_empty : context := Context.empty type.
Inductive expr : Set :=
| eunit : expr
| evar : var -> expr
| eabs : var -> type -> expr -> expr
| eapp : expr -> expr -> expr.
Fixpoint free_vars (e : expr) : VarSet.t :=
match e with
| eunit => VarSet.empty
| evar y => VarSet.singleton y
| eabs y _ e => VarSet.remove y (free_vars e)
| eapp e1 e2 => VarSet.union (free_vars e1) (free_vars e2)
end.
Inductive has_type : context -> expr -> type -> Prop :=
| has_type_unit : forall c,
has_type c eunit tunit
| has_type_var : forall c x t,
Context.find x c = Some t ->
has_type c (evar x) t
| has_type_abs : forall c x t1 t2 e,
has_type (Context.add x t1 c) e t2 ->
has_type c (eabs x t1 e) (tfun t1 t2)
| has_type_app : forall c e1 e2 t1 t2,
has_type c e1 (tfun t1 t2) ->
has_type c e2 t1 ->
has_type c (eapp e1 e2) t2.
Check has_type_ind.
Lemma has_type_empty_context_free_vars : forall e t,
has_type context_empty e t ->
VarSet.Empty (free_vars e).
Proof.
intros e t H.
remember context_empty as c.
induction H; subst.
- apply VarSet.empty_spec.
- rewrite ContextFacts.empty_o in H.
congruence.
- simpl.
admit. (* Wrong induction hypothesis *)
- simpl.
rewrite VarSetProps.empty_union_1; auto.
Admitted.
问题似乎是我的归纳假设是错误的。它只是说
Context.add x t1 context_empty = context_empty ->
VarSet.Empty (free_vars e)
这很简单,因为这个假设是错误的。我试着对表达式进行归纳并重新定义该定理以获得正确的归纳假设,但无法弄明白。
定义和证明此属性的正确方法是什么?
继Yves'answer之后,感谢ejgallego的评论,我首先证明了一个普遍的引理。
Lemma has_type_free_vars_in_context : forall c e t,
has_type c e t ->
VarSet.For_all (fun x => Context.mem x c = true) (free_vars e).
Proof.
intros c e t H.
induction H; simpl.
- intros x contra.
apply VarSetFacts.empty_iff in contra.
inversion contra.
- intros y H2.
apply Context.mem_1.
apply ContextFacts.in_find_iff.
apply VarSet.singleton_spec in H2.
subst.
rewrite H.
discriminate.
- intros y H2.
unfold VarSet.For_all in *.
apply VarSet.remove_spec in H2 as [H2 H3].
specialize (IHhas_type y H2).
rewrite ContextFacts.add_neq_b in IHhas_type; auto.
- intros x H2.
apply VarSet.union_spec in H2 as [H2 | H2]; auto.
Qed.
曾经用它来证明我的定理。
Lemma has_type_empty_context_free_vars : forall e t,
has_type context_empty e t ->
VarSet.Empty (free_vars e).
Proof.
intros e t H.
apply has_type_free_vars_in_context in H.
induction (free_vars e) using VarSetProps.set_induction.
- assumption.
- rename t0_1 into s.
rename t0_2 into s'.
apply VarSetProps.Add_Equal in H1.
unfold VarSet.For_all in *.
specialize (H x).
rewrite H1 in H.
specialize (H (VarSetFacts.add_1 s eq_refl)).
Search (Context.empty).
rewrite ContextFacts.empty_a in H.
discriminate.
Qed.
它现在有效。非常感谢你。有没有办法重构这个解决方案,以实现更高的自动化,更好的可读性,更好的维护等等?
答案 0 :(得分:3)
你对声明" has_type ..."的假设进行归纳是正确的,但你可能需要加载归纳法。换句话说,您需要证明一个更强的语句,使环境变量,并表示e
中的自由变量集必须位于您的上下文中具有类型的变量内。