Coq:本地ltac定义

Coq:本地ltac定义,coq,ltac,Coq,Ltac,如果有一种方法可以定义一个“本地”Ltac表达式,我可以用它来证明一个引理,但在外面看不见 Lemma Foo ... Proof. Ltac ll := ... destrict t. - reflexivity. - ll. - ll. Qed. (* ll should not be visible here *) 您可以使用以下部分: Section Foo. Ltac solve := exact I. Lemma Foo : True.

如果有一种方法可以定义一个“本地”Ltac表达式,我可以用它来证明一个引理,但在外面看不见

Lemma Foo ...
Proof.
   Ltac ll := ...
   destrict t.
   - reflexivity.
   - ll.
   - ll.
Qed.

(* ll should not be visible here *)
您可以使用以下部分:

Section Foo.
  Ltac solve := exact I.
  Lemma Foo : True.
  Proof.
    solve.
  Qed.
End Foo.