我被卡在一個目標上。 假設我們有如下定義: Fixpoint iota (n : nat) : list nat :=
match n with
| 0 => []
| S k => iota k ++ [k]
end.
我們要證明: Theorem t1 : forall n, In n (iota n) -> False. 到目前爲止,我已成功地執行
給定集合包含的證明及其相反,我希望能夠證明兩個集合是平等的。 例如,我知道如何證明following statement,並its converse: open set
universe u
variable elem_type : Type u
variable A : set elem_type
variable B : set elem_type
def set_deMorga
我想通過z3來證明(∀i(0≤i<k→a[i]>0)∧a[k]>0)→∀i(0≤i≤k→a[i]>0)。否定它是:∀i(0≤i<k→a[i]>0)∧a[k]>0∧∃i(0≤i≤k∧¬(a[i]>0))。首先,我k的值設置爲5,而忽略部分a[k]>0,並嘗試: from z3 import *
i = Int('i')`
a = Array('a',IntSort(),IntSort())
s