Theory AxLightMinus
section ‹ AXIOM: AxLightMinus ›
text ‹This theory declares the axiom AxLightMinus.›
theory AxLightMinus
imports WorldLine TangentLines
begin
text ‹AxLightMinus:
If an observer sends out a light signal, then the speed of the
light signal is 1 according to the observer. Moreover it is possible to send
out a light signal in any direction.›
class axLightMinus = WorldLine + TangentLines
begin
text ‹The definition of AxLightMinus used in this Isabelle proof is slightly
different to the one used in the paper-based proof on which it is based. We
have established elsewhere, however, that each entails the other in all
relevant contexts.›
abbreviation axLightMinusOLD :: "Body ⇒ 'a Point ⇒ 'a Space ⇒ bool"
where "axLightMinusOLD m p v ≡ (m sees m at p) ⟶ (
(∃ ph . (Ph ph ∧ (vel (wline m ph) p v))) ⟷ (sNorm2 v = 1)
)"
abbreviation axLightMinus :: "Body ⇒ 'a Point ⇒ 'a Space ⇒ bool"
where "axLightMinus m p v ≡ (m sees m at p)
⟶ ( ∀ l . ∀ v ∈ lineVelocity l .
(∃ ph . (Ph ph ∧ (tangentLine l (wline m ph) p))) ⟷ (sNorm2 v = 1))"
end
class AxLightMinus = axLightMinus +
assumes AxLightMinus: "∀ m p v . axLightMinus m p v"
begin
end
end