Skip to content

Commit

Permalink
FTBFS
Browse files Browse the repository at this point in the history
  • Loading branch information
binghe committed Nov 30, 2024
1 parent ebc5248 commit 126391b
Showing 1 changed file with 3 additions and 1 deletion.
4 changes: 3 additions & 1 deletion src/boss/prove_base_assumsScript.sml
Original file line number Diff line number Diff line change
Expand Up @@ -424,6 +424,8 @@ val th2 = store_thm
("th2", el 2 goals |> concl,
rpt gen_tac \\ MATCH_ACCEPT_TAC (CONJ (SPEC_ALL if_T) (SPEC_ALL if_F)));

val bool_case_lemma = th2;

val cons_11 = hd (amatch ``Data_List_cons _ _ = Data_List_cons _ _``);

(* |- !a0 a1 a0' a1'.
Expand Down Expand Up @@ -1635,7 +1637,7 @@ val BOOL_EQ_DISTINCT = store_thm("BOOL_EQ_DISTINCT", concl boolTheory.BOOL_EQ_DI
*)
val bool_case_thm = store_thm
("bool_case_thm", concl boolTheory.bool_case_thm,
PURE_REWRITE_TAC[th18]
PURE_REWRITE_TAC[bool_case_lemma]
\\ conj_tac \\ rpt gen_tac \\ REFL_TAC);

val forall_bool = hd(amatch``(!b:bool. P b) <=> _``)
Expand Down

0 comments on commit 126391b

Please sign in to comment.