微信公众号搜"智元新知"关注
微信扫一扫可直接关注哦!

是否可以在 Isabelle 的函数域中添加假设?

如何解决是否可以在 Isabelle 的函数域中添加假设?

我不确定是否可以发布这样的后续问题,但我还是会这样做。

所以几天前我发布了这个问题:How can I remove all occurrences of a sub-multiset in Isabelle?

我认为答案很好,但是在尝试证明引理时

lemma "applied1 {#''a'',''a'',''d'',''c'',''c''#} {#''a'',''c''#} ''f'' = {#''f'',''f'',''d''#}"

我真的卡住了。我发现在展开 def 并应用一些简单的自动化之后,我不能简单地做到这一点。所以我回到我原来的函数并对其进行了一些调整,这样如果输入导致无限循环,它就不返回任何内容。我以为这次会奏效,但伊莎贝尔仍然无法证明终止。我很确定很明显 size x 不断减少 size y 的因子并且不能为负,因此它最终必须在 size x = 0 或当 y 不再是x 的子集。

fun applied2 :: "'a multiset ⇒ 'a multiset ⇒ 'a ⇒ 'a multiset option" where
"applied2 x y z = (if z ∈# y ∨ y = {#} then None else (if y ⊆# x then Some (plus {#z#} (the (applied2 (x - y) y z))) else Some x))"

是否可以让 Isabelle 相信此函数使用 function 而不是 fun 终止?或者我还需要考虑其他限制吗?

如果我不应该发布这样的问题,我真的很抱歉。我对伊莎贝尔仍然缺乏经验,我确实希望我能坚持我的目标,尽我所能地学习这门语言。提前致谢!

解决方法

我相信查看 documentation 会为您提供正确的语法。

function applied2 :: "'a multiset ⇒ 'a multiset ⇒ 'a ⇒ 'a multiset option" where
"applied2 x y z = (if z ∈# y ∨ y = {#} then None else (if y ⊆# x then Some (plus {#z#} (the (applied2 (x - y) y z))) else Some x))"
  by pat_completeness auto
termination
  by (relation "measure (λ(x,y,z). size x)")
    (auto simp: mset_subset_eq_exists_conv nonempty_has_size)

如果问题是证据,大锤会帮你找到的。

但是,我不明白您打算如何从应用 2 转到您真正想要的功能。真正的问题是确定性:您需要一个命令来查看子集。 Manuel 的解决方案是使用 Sup,但这确实无法执行。

,

如果非递归定义的唯一问题是如何将其应用于具体输入,我仍然认为我所说的可执行的替代定义是可行的方法。这里证明我给出的两个非递归定义是等价的,以及你上面给出的例子的应用:

definition applied :: "'a multiset ⇒ 'a multiset ⇒ 'a ⇒ 'a multiset" where
  "applied ms xs y = (if xs = {#} then ms else
     (let n = Max {n. repeat_mset n xs ⊆# ms}
      in ms - repeat_mset n xs + replicate_mset n y))"

lemma count_le_size: "count M x ≤ size M"
  by (induction M) auto

lemma applied_code [code]:
  "applied ms xs y = (if xs = {#} then ms else
     (let n = (MIN x ∈set_mset xs. count ms x div count xs x)
      in ms - repeat_mset n xs + replicate_mset n y))"
  unfolding applied_def
proof (intro if_cong let_cong refl)
  assume ne: "xs ≠ {#}"
  have subset: "{n. repeat_mset n xs ⊆# ms} ⊆ {..size ms}"
  proof safe
    fix n assume n: "repeat_mset n xs ⊆# ms"
    from ne obtain x where x: "x ∈# xs"
      by auto
    have "n * 1 ≤ n * count xs x"
      using x by (intro mult_left_mono) auto
    also have "… = count (repeat_mset n xs) x"
      by simp
    also have "… ≤ count ms x"
      using n by (intro mset_subset_eq_count)
    also have "… ≤ size ms"
      by (rule count_le_size)
    finally show "n ≤ size ms" by simp
  qed
  hence finite: "finite {n. repeat_mset n xs ⊆# ms}"
    by (rule finite_subset) auto

  show "Max {n. repeat_mset n xs ⊆# ms} = (MIN x∈set_mset xs. count ms x div count xs x)"
  proof (intro antisym)
    show "Max {n. repeat_mset n xs ⊆# ms} ≤ (MIN x∈set_mset xs. count ms x div count xs x)"
    proof (rule Max.boundedI)
      show "{n. repeat_mset n xs ⊆# ms} ≠ {}"
        by (auto intro: exI[of _ 0])
    next
      fix n assume n: "n ∈ {n. repeat_mset n xs ⊆# ms}"
      show "n ≤ (MIN x∈set_mset xs. count ms x div count xs x)"
      proof (safe intro!: Min.boundedI)
        fix x assume x: "x ∈# xs"
        have "count (repeat_mset n xs) x ≤ count ms x"
          using n by (intro mset_subset_eq_count) auto
        also have "count (repeat_mset n xs) x = n * count xs x"
          by simp
        finally show "n ≤ count ms x div count xs x"
          by (metis count_eq_zero_iff div_le_mono nonzero_mult_div_cancel_right x)
      qed (use ne in auto)
    qed (fact finite)
  next
    define m where "m = (MIN x∈set_mset xs. count ms x div count xs x)"
    show "m ≤ Max {n. repeat_mset n xs ⊆# ms}"
    proof (rule Max.coboundedI[OF finite],safe)
      show "repeat_mset m xs ⊆# ms"
      proof (rule mset_subset_eqI)
        fix x
        show "count (repeat_mset m xs) x ≤ count ms x"
        proof (cases "x ∈# xs")
          case True
          have "count (repeat_mset m xs) x = m * count xs x"
            by simp
          also have "… ≤ (count ms x div count xs x) * count xs x"
            unfolding m_def using ‹x ∈# xs› by (intro mult_right_mono Min.coboundedI) auto
          also have "… ≤ count ms x"
            by simp
          finally show ?thesis .
        next
          case False
          hence "count xs x = 0"
            by (meson not_in_iff)
          thus ?thesis by simp
        qed
      qed
    qed
  qed
qed

lemma replicate_mset_unfold:
  assumes "n > 0"
  shows   "replicate_mset n x = {#x#} + replicate_mset (n - 1) x"
  using assms by (cases n) auto

lemma
  assumes "a ≠ c" "a ≠ f" "c ≠ f"
  shows   "applied {#a,a,c,c#} {#a,c#} f = mset [f,f]"
  using assms
  by (simp add: applied_code replicate_mset_unfold flip: One_nat_def)

value 命令不适用于该示例,因为 ac 等是自由变量。但是如果你例如为他们制作一个特别的数据类型,它可以工作:

datatype test = a | b | c | f

value "applied {#a,c#} f"
(* "mset [f,f]" :: "test multiset" *)

版权声明:本文内容由互联网用户自发贡献,该文观点与技术仅代表作者本人。本站仅提供信息存储空间服务,不拥有所有权,不承担相关法律责任。如发现本站有涉嫌侵权/违法违规的内容, 请发送邮件至 dio@foxmail.com 举报,一经查实,本站将立刻删除。