Skip to content

Commit

Permalink
Fix error in nfmbstScript.sml
Browse files Browse the repository at this point in the history
  • Loading branch information
mn200 committed Sep 13, 2023
1 parent 99b8c21 commit 63228ef
Showing 1 changed file with 8 additions and 8 deletions.
16 changes: 8 additions & 8 deletions src/transfer/examples/nfmbstScript.sml
Original file line number Diff line number Diff line change
Expand Up @@ -349,14 +349,6 @@ Proof
simp[NFMBST_def] >> metis_tac[FAPPLY_bst_to_fm]
QED

Theorem NFMfoo[transfer_rule]:
((=) |==> NFMBST (=)) foo foo'
Proof
simp[FUN_REL_def, foo'_def] >> gen_tac >> SELECT_ELIM_TAC >> conj_tac
>- metis_tac[bst_to_fm_surj] >>
simp[NFM_bst_to_fm]
QED

Theorem NFMEQ[transfer_rule]:
(NFMBST (=) |==> NFMBST (=) |==> flip (==>)) (=) (=)
Proof
Expand All @@ -374,6 +366,14 @@ Definition foo'_def:
foo' n = @bst. bst_to_fm bst = foo n /\ wfBST bst
End
Theorem NFMfoo[transfer_rule]:
((=) |==> NFMBST (=)) foo foo'
Proof
simp[FUN_REL_def, foo'_def] >> gen_tac >> SELECT_ELIM_TAC >> conj_tac
>- metis_tac[bst_to_fm_surj] >>
simp[NFM_bst_to_fm]
QED
*)


Expand Down

0 comments on commit 63228ef

Please sign in to comment.