Skip to content

Commit 686f85a

Browse files
committed
Fix breakage
1 parent 38841a7 commit 686f85a

File tree

5 files changed

+19
-19
lines changed

5 files changed

+19
-19
lines changed

examples/lambda/barendregt/boehmScript.sml

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1058,7 +1058,7 @@ Proof
10581058
>> reverse (Cases_on ‘solvable M’)
10591059
>- rw [subterm_def, BT_of_unsolvables, ltree_el_def]
10601060
(* stage work *)
1061-
>> rw [subterm_def, BT_def, BT_generator_def, Once ltree_unfold, ltree_el_def]
1061+
>> simp[subterm_def, BT_def, BT_generator_def, Once ltree_unfold, ltree_el_def]
10621062
>> qabbrev_tac ‘M0 = principle_hnf M’
10631063
>> qabbrev_tac ‘n = LAMl_size M0’
10641064
>> Q_TAC (RNEWS_TAC (“vs :string list”, “r :num”, “n :num”)) ‘X’

examples/lambda/barendregt/normal_orderScript.sml

Lines changed: 2 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -188,7 +188,8 @@ val bnf_noposn = store_thm(
188188
"bnf_noposn",
189189
``∀M. bnf M ⇔ (noposn M = NONE)``,
190190
HO_MATCH_MP_TAC simple_induction THEN
191-
SRW_TAC [][] THEN Cases_on `noposn M` THEN SRW_TAC [][])
191+
SRW_TAC [][] THEN Cases_on `noposn M` THEN
192+
SRW_TAC [][EQ_IMP_THM])
192193

193194
val normorder_noposn = store_thm(
194195
"normorder_noposn",

src/finite_maps/alist_treeScript.sml

Lines changed: 3 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -307,11 +307,10 @@ Theorem is_lookup_far_left:
307307
!R k k' v. R k k' ==> is_lookup F T R [(k', v)] k NONE
308308
Proof
309309
fs [is_lookup_def, sortingTheory.SORTED_EQ, listTheory.MEM_MAP,
310-
pairTheory.EXISTS_PROD]
310+
pairTheory.EXISTS_PROD,alistTheory.ALOOKUP_NONE,PULL_EXISTS]
311311
\\ rpt strip_tac
312-
\\ Cases_on `ALOOKUP ys k` \\ CASE_TAC \\ fs []
313-
\\ metis_tac [alistTheory.ALOOKUP_MEM, relationTheory.irreflexive_def,
314-
relationTheory.transitive_def]
312+
\\ metis_tac [ relationTheory.irreflexive_def,
313+
relationTheory.transitive_def]
315314
QED
316315

317316
Theorem is_lookup_far_right:

src/pred_set/src/more_theories/cardinalScript.sml

Lines changed: 4 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -3178,13 +3178,13 @@ Proof
31783178
else if (!x. x IN s ==> ISR x) /\ IMAGE OUTR s IN As then
31793179
SOME (INR (THE (SND p (IMAGE OUTR s))))
31803180
else NONE’ >>
3181-
rw[] >> simp[AllCaseEqs(), PULL_EXISTS]
3181+
rw[] >> simp[PULL_EXISTS]
31823182
>- (metis_tac[THE_DEF, MEMBER_NOT_EMPTY])
31833183
>- (rename [‘s = {}’, ‘s <> IMAGE INL A’] >>
3184-
pop_assum mp_tac >> rw[]
3184+
rpt (IF_CASES_TAC >> fs[])
31853185
>- (qpat_x_assum ‘s <> IMAGE INL _’ mp_tac >>
3186-
csimp[EXTENSION, PULL_EXISTS, sumTheory.INL]) >>
3187-
first_x_assum $ qspec_then ‘IMAGE OUTR s’ mp_tac >> simp[]) >>
3186+
rw[CONTRAPOS_THM] >> gvs[]) >>
3187+
fs[DISJ_EQ_IMP]) >>
31883188
qexists_tac ‘λtup. (OUTL (THE (tup (IMAGE INL A))),
31893189
(λB. if B IN As then
31903190
SOME (OUTR (THE (tup (IMAGE INR B))))

src/pred_set/src/more_theories/wellorderScript.sml

Lines changed: 9 additions & 9 deletions
Original file line numberDiff line numberDiff line change
@@ -595,15 +595,15 @@ val wo2wo_EQ_NONE = store_thm(
595595
``!x. (wo2wo w1 w2 x = NONE) ==>
596596
!y. (x,y) WIN w1 ==> (wo2wo w1 w2 y = NONE)``,
597597
ONCE_REWRITE_TAC [wo2wo_thm] >> rw[LET_THM] >>
598-
match_mp_tac SUBSET_ANTISYM >> rw[IMAGE_wo2wo_SUBSET] >>
599-
match_mp_tac SUBSET_TRANS >>
600-
qexists_tac `IMAGE THE (IMAGE (wo2wo w1 w2) (iseg w1 x) DELETE NONE)` >>
601-
conj_tac >- (
602-
Cases_on`wleast w2 (IMAGE THE (IMAGE (wo2wo w1 w2) (iseg w1 x) DELETE NONE))` >>
603-
imp_res_tac wleast_EQ_NONE >> fs[] ) >>
604-
simp_tac (srw_ss() ++ DNF_ss) [SUBSET_DEF] >>
605-
qsuff_tac `!a. a IN iseg w1 x ==> a IN iseg w1 y` >- metis_tac[] >>
606-
rw[iseg_def] >> metis_tac [WIN_TRANS]);
598+
fs[IMAGE_wo2wo_SUBSET,SET_EQ_SUBSET]
599+
>- (
600+
qsuff_tac `elsOf w2 ⊆ IMAGE THE (IMAGE (wo2wo w1 w2) (iseg w1 y) DELETE NONE)` >- fs[] >>
601+
MATCH_MP_TAC SUBSET_TRANS >>
602+
first_x_assum (irule_at (Pos hd)) >>
603+
simp_tac (srw_ss() ++ DNF_ss) [SUBSET_DEF] >>
604+
qsuff_tac `!a. a IN iseg w1 x ==> a IN iseg w1 y` >- metis_tac[] >>
605+
rw[iseg_def] >> METIS_TAC[WIN_TRANS])
606+
>- imp_res_tac wleast_EQ_NONE);
607607

608608
val wo2wo_EQ_SOME_downwards = store_thm(
609609
"wo2wo_EQ_SOME_downwards",

0 commit comments

Comments
 (0)