Isabelle中是否有重写策略?

问题描述 投票:3回答:1

例如,在Coq中有rewrite,我们也可以放箭头`

Inductive bool: Set :=
  | true
  | false.

Lemma equality_of_functions_commutes:
  forall (f: bool->bool) x y,
    (f x) = (f y) -> (f y) = (f x).
Proof.
  intros.
  rewrite H.
  reflexivity.
Qed.

来源:https://pjreddie.com/coq-tactics/#rewrite

isabelle theorem-proving
1个回答
2
投票

我不认为它与Coq版本一样强大,但是

重写定理。但是,您无法轻松地以应用样式重写假设。

© www.soinside.com 2019 - 2024. All rights reserved.