~~/src/HOL/Word/Word.thy中有一個稱爲word_rsplit的功能。 definition word_rsplit :: "'a :: len0 word => 'b :: len word list" where
"word_rsplit w =
map word_of_int (bin_rsplit (len_of TYPE ('b)) (len_of
我已經試過證明樂趣bubble_main是有序的,但沒有辦法似乎工作。請問這裏有人能幫我證明引理is_ordered (bubble_main L)。 我剛剛刪除了我以前的所有引理,因爲似乎沒有任何幫助Isabelle找到一個證明。 這裏是我的代碼/理論:所有的 text{*check if the list is ordered ascendant*}
fun is_sorted :: "na
我試圖證明如下含義: lemma Max_lemma:
fixes s::nat and S :: "nat set"
shows " ((Max S) = (0::nat)) ⟹ (∀ s ∈ S . (s = 0))"
sorry
(*
Note: I added additional parentheses just to be sure.*)
我想這將
我試圖使用轉移包爲自定義數據類型建立歸納規則,但apply transfer不適用於我。下面是一個簡單的例子: theory TransferHO imports Main begin
typedef pos = "{x :: nat. x > 0}" by blast
setup_lifting type_definition_pos
lift_definition one :: po