考虑以下愚蠢的Isabelle对树和子树的定义:
datatype tree = Leaf int
| Node tree tree
fun children :: "tree ⇒ tree set" where
"children (Leaf _) = {}" |
"children (Node a b) = {a, b}"
lemma children_decreasing_size:
assumes "c ∈ children t"
shows "size c < size t"
using assms
by (induction t, auto)
function subtrees :: "tree ⇒ tree set" where
"subtrees t = { s | c s. c ∈ children t ∧ s ∈ subtrees c }"
by auto
termination
apply (relation "measure size", simp)
subtrees
的终止证明在这一点上被卡住了,尽管递归调用只是针对儿童进行的,这些儿童严格按照有充分根据的size
关系进行调整(正如琐碎的引理所示)
证明状态如下:
goal (1 subgoal):
1. ⋀t x xa xb. (xa, t) ∈ measure size
当然,这是不可能证明的,因为xa
是t
的孩子的信息丢失了。我做错什么了吗?我能做些什么来保存证明吗?我注意到我可以使用列表而不是集来制定相同的定义:
fun children_list :: "tree ⇒ tree list" where
"children_list (Leaf _) = []" |
"children_list (Node a b) = [a, b]"
function subtrees_list :: "tree ⇒ tree list" where
"subtrees_list t = concat (map subtrees_list (children_list t))"
by auto
termination
apply (relation "measure size", simp)
并获得更具信息性,可证明的终止目标:
goal (1 subgoal):
1. ⋀t x.
x ∈ set (children_list t) ⟹
(x, t) ∈ measure size
这是Isabelle的一些限制,我应该通过不使用套装来解决这个问题吗?
答案 0 :(得分:3)
对c : children t
的集合理解中subtrees
的限制未出现在终止证明义务中,因为函数包对&
的先验不知道。同余规则可用于实现此目的。在这种情况下,您可以在本地将conj_cong
声明为[fundef_cong]
,以基本上模拟从左到右的评估顺序(尽管在HOL中没有评估这样的事情)。例如,
context notes conj_cong[fundef_cong] begin
fun subtrees :: ...
termination ...
end
上下文块确保声明conj_cong[fundef_cong]
仅对此函数定义有效。
包含列表的版本之所以有效,是因为它使用的函数map
默认情况下存在同余规则。如果您在集合上使用了monadic绑定操作(而不是集合理解),那么对于集合应该也适用。