jrh13 / hol-light

The HOL Light theorem prover
Other
435 stars 79 forks source link

unnecessary hyp in TAN_ADD #63

Closed thery closed 3 years ago

thery commented 3 years ago

in transc.ml lime 2605 : let TAN_ADD = prove( !x y. ~(cos(x) = &0) /\ ~(cos(y) = &0) /\ ~(cos(x + y) = &0) ==> (tan(x + y) = (tan(x) + tan(y)) / (&1 - tan(x) * tan(y))),

the assumption ~(cos(x + y) = &0) seems unnecessary.

thery commented 3 years ago

my bad, you don't have inv(0) = 0