Skip to content

Commit

Permalink
Add cv_rep for fEMPTY: num_set
Browse files Browse the repository at this point in the history
  • Loading branch information
xrchz committed Oct 9, 2024
1 parent 5c52458 commit 4821902
Showing 1 changed file with 11 additions and 0 deletions.
11 changes: 11 additions & 0 deletions src/num/theories/cv_compute/automation/cv_stdScript.sml
Original file line number Diff line number Diff line change
Expand Up @@ -472,9 +472,20 @@ Proof
GSYM fIN_IN, domain_list_to_num_set, fIN_def]
QED

val from_sptree_sptree_spt_def = definition "from_sptree_sptree_spt_def";
val cv_insert_thm = theorem "cv_insert_thm";
val cv_lookup_thm = theorem "cv_lookup_thm";

Theorem fEMPTY_num_cv_rep[cv_rep]:
from_num_fset fEMPTY = Num 0
Proof
rw[from_num_fset_def,
Q.ISPEC`from_unit`(CONJUNCT1(GSYM from_sptree_sptree_spt_def))]
\\ AP_TERM_TAC
\\ DEP_REWRITE_TAC[spt_eq_thm]
\\ rw[lookup_list_to_num_set, wf_list_to_num_set, MEM_fset_REP]
QED

Theorem fINSERT_num_cv_rep[cv_rep]:
from_num_fset (fINSERT e s) =
cv_insert (Num e) (Num 0) (from_num_fset s)
Expand Down

0 comments on commit 4821902

Please sign in to comment.