Skip to content

Commit

Permalink
Style tweaks to last commit
Browse files Browse the repository at this point in the history
See also Github PR #1008.

Change to use modern syntax, and remove redundant calls to `simp`.
  • Loading branch information
mn200 committed Jan 11, 2023
1 parent 02db589 commit 21546e9
Showing 1 changed file with 5 additions and 7 deletions.
12 changes: 5 additions & 7 deletions src/floating-point/binary_ieeeScript.sml
Expand Up @@ -4166,16 +4166,14 @@ val float_div_minus_infinity_finite = Q.store_thm(

(* - - - - - - - - - - - - - - - - - - - - - - - - - - - - - - - - - - - - *)

val float_is_nan_impl = Q.store_thm(
"float_is_nan_impl",
`!x. float_is_nan x <=> ~float_equal x x`,
Theorem float_is_nan_impl:
!x. float_is_nan x <=> ~float_equal x x
Proof
simp[float_is_nan_def, float_equal_def, float_compare_def]
\\ STRIP_TAC
\\ strip_tac
\\ Cases_on `float_value x`
\\ simp[]
\\ simp[]
\\ simp[]
)
QED

(* ------------------------------------------------------------------------ *)

Expand Down

0 comments on commit 21546e9

Please sign in to comment.