Skip to content

Commit b34f7b7

Browse files
committed
Fix proofs after reln type abbrev was properly removed
1 parent fa6973c commit b34f7b7

File tree

1 file changed

+5
-5
lines changed

1 file changed

+5
-5
lines changed

lca/lcaProofScript.sml

+5-5
Original file line numberDiff line numberDiff line change
@@ -2057,7 +2057,7 @@ val termsem_strong_limit_cardinal = store_thm("termsem_strong_limit_cardinal",
20572057
simp[Abbr`vvx`,APPLY_UPDATE_THM] >>
20582058
simp[Abbr`vv`,Abbr`s`,APPLY_UPDATE_THM,UPDATE_LIST_THM] >>
20592059
CONV_TAC(LAND_CONV(REWR_CONV inter_subset)) >>
2060-
Q.PAT_ABBREV_TAC`P:'U set reln = $SUBSET` >>
2060+
Q.PAT_ABBREV_TAC`P:'U set -> 'U set -> bool = $SUBSET` >>
20612061
simp[Holds_Abstract,boolean_in_boolset] >>
20622062
simp[Abbr`P`,boolean_eq_true] >>
20632063
simp[SUBSET_DEF,IN_DEF] ) >>
@@ -2120,7 +2120,7 @@ val termsem_strong_limit_cardinal = store_thm("termsem_strong_limit_cardinal",
21202120
simp[Holds_Abstract,boolean_in_boolset] >>
21212121
simp[boolean_eq_true] >>
21222122
ONCE_REWRITE_TAC[inter_subset] >>
2123-
Q.PAT_ABBREV_TAC`P:'U set reln = $SUBSET` >>
2123+
Q.PAT_ABBREV_TAC`P:'U set -> 'U set -> bool = $SUBSET` >>
21242124
simp[Holds_Abstract,boolean_in_boolset] >>
21252125
simp[Abbr`P`,boolean_eq_true] >>
21262126
simp[Abbr`vv`,APPLY_UPDATE_THM,UPDATE_LIST_THM,Abbr`s`] >>
@@ -2820,7 +2820,7 @@ val LCA_name_UNIV = replace_term ``strlit"l"``name LCA_l_UNIV
28202820
val intermediate_thm_gen = Q.store_thm("intermediate_thm_gen",
28212821
`(name ≠ strlit"f" ∧ name ≠ strlit"k") (* makes proof easier *)
28222822
LCA (SUC l) (UNIV:'U set) ⇒
2823-
∃(mem:'U reln).
2823+
∃(mem:'U -> 'U -> bool).
28242824
is_set_theory mem ∧ (∃inf. is_infinite mem inf) ∧
28252825
wf_to_inner ((to_inner Ind):ind->'U) ∧
28262826
(wf_to_inner ((to_inner_Num mem):num->'U) ∧
@@ -3198,7 +3198,7 @@ val intermediate_thm_gen = Q.store_thm("intermediate_thm_gen",
31983198
qmatch_abbrev_tac`A ∩ B ⊆ C` >>
31993199
`A ∩ B ⊆ A ∩ C` suffices_by simp[] >>
32003200
map_every qunabbrev_tac[`A`,`B`,`C`] >>
3201-
Q.PAT_ABBREV_TAC`P:'U set reln = $SUBSET` >>
3201+
Q.PAT_ABBREV_TAC`P:'U set -> 'U set -> bool = $SUBSET` >>
32023202
simp[Holds_Abstract,boolean_in_boolset] >>
32033203
simp[Abbr`P`,boolean_eq_true] >>
32043204
fs[SUBSET_DEF] >>
@@ -3257,7 +3257,7 @@ val intermediate_thm_gen = Q.store_thm("intermediate_thm_gen",
32573257
val intermediate_thm = store_thm("intermediate_thm",
32583258
``(name ≠ strlit"f" ∧ name ≠ strlit"k") (* makes proof easier *)
32593259
LCA (SUC l) (UNIV:'U set) ⇒
3260-
∃(mem:'U reln).
3260+
∃(mem:'U -> 'U -> bool).
32613261
is_set_theory mem ∧ (∃inf. is_infinite mem inf) ∧
32623262
wf_to_inner ((to_inner Ind):ind->'U) ∧
32633263
(wf_to_inner ((to_inner Num):num->'U) ∧

0 commit comments

Comments
 (0)