Skip to content

Commit

Permalink
Use cv_trans instead of cv_trans_pre in a few places
Browse files Browse the repository at this point in the history
  • Loading branch information
myreen committed Apr 4, 2024
1 parent 4d623c3 commit 2875e0c
Showing 1 changed file with 4 additions and 4 deletions.
8 changes: 4 additions & 4 deletions src/num/theories/cv_compute/automation/cv_stdScript.sml
Original file line number Diff line number Diff line change
Expand Up @@ -185,12 +185,12 @@ QED
val all_distinct =
ALL_DISTINCT |> DefnBase.one_line_ify NONE |> PURE_REWRITE_RULE [conj_eq_if,if_not]

val res = cv_trans_pre all_distinct;
val res = cv_trans all_distinct;

val is_prefix =
isPREFIX |> DefnBase.one_line_ify NONE |> PURE_REWRITE_RULE [conj_eq_if,if_not]

val res = cv_trans_pre is_prefix;
val res = cv_trans is_prefix;

val res = cv_trans LUPDATE_DEF;

Expand All @@ -209,7 +209,7 @@ Proof
\\ rename [‘_ = SOME y’] \\ PairCases_on ‘y’ \\ gvs []
QED

val res = cv_trans_pre index_of
val res = cv_trans_pre index_of;

Definition replicate_acc_def:
replicate_acc n x acc =
Expand Down Expand Up @@ -248,7 +248,7 @@ Proof
\\ gvs [UNZIP] \\ Cases_on ‘UNZIP t’ \\ gvs []
QED

val res = cv_trans_pre UNZIP_eq
val res = cv_trans UNZIP_eq

Definition genlist_def:
genlist i f 0 = [] /\
Expand Down

0 comments on commit 2875e0c

Please sign in to comment.