my_inductive_intros
我们可以用更漂亮的basecase和默认stepcase定义一组新的引入规则
lemma my_inductive_intro_1: "my_inductive (a, b) a"
by (simp add: my_inductive.basecase)
lemmas my_inductive_intros = my_inductive_intro_1 my_inductive.stepcase
我们可以编写自己漂亮的归纳规则
lemma my_inductive_tuple_induct[consumes 1, case_names "basecase" "stepcase", induct pred: my_inductive]:
"my_inductive (a, b) x ⟹
(P a) ⟹ (⋀x y. someP (a, b) x y ⟹ my_inductive (a, b) x ⟹ P x ⟹ P y) ⟹ P x"
apply(rule my_inductive.induct[of "(a,b)"])
apply(simp_all)
done
consumes 1
告诉 isabelle 使用第一个参数。让我们通过一个例子来说明这一点:
lemma "my_inductive (a,b) c ⟹ P a b c"
proof(induction rule: my_inductive_tuple_induct)
没有[consumes 1]
这个就是证明状态:
- my_inductive (?a, ?b) (my_inductive (a, b) c ⟶ P abc)
- ?一种
- ⋀xy。someP (?a, ?b) xy ⟹ my_inductive (?a, ?b) x ⟹ x ⟹ y
有了[consumes 1]
,我们得到了想要的证明状态:
- 爸爸
- ⋀xy。someP (a, b) xy ⟹ my_inductive (a, b) x ⟹ P abx ⟹ P aby
case_names
为 isar 证明设置案例名称。因此,上述证明可以从 开始case basecase
。
induct pred
告诉我们正在声明一个归纳规则。在某些情况下,proof(induction)
现在仅仅写作可能就足以让 isabelle 自己找出来使用我们新的奇特归纳规则。
以下示例演示了设置
lemma
assumes "my_inductive (a,b) c" shows "P a b c"
using assms
proof (induction)
case basecase thus ?case using my_inductive_intros sorry
case (stepcase x y) thus ?case using my_inductive_intros sorry
qed