了解 Isabelle 中的导数(“在 .. 之内”的意思)
Understanding derivatives in Isabelle (meaning of `at .. within`)
这是一个关于 Isabelle 库中导数概念的问题。
我正在尝试理解 (f has_field_derivative D x) (at x within S)
的含义。我知道 (at x within S)
是一个过滤器,但直觉上我在想下面的语句是真的
lemma DERIV_at_within:
"(∀x ∈ S. (f has_field_derivative D x) (at x))
= (∀x. (f has_field_derivative D x) (at x within S))"
如果不是,我还应该如何解释 (at x within S)
在导数的上下文中?
at x within A
是x
的尖邻域,与A
相交。例如,at_right
是at x within {x<..}
的缩写,即x
的右邻域。这允许您表达单边导数。
偶尔也会看到像∀x∈{a..b}. (f has_field_derivative f' x) (at x within {a..b})
这样的假设。这意味着 f
与导数 f'
在 a
和 b
之间是可微的,但是边缘处的导数(即在 a
和 b
) 只需要是单方面的。
另请注意 at x = at x within UNIV
。此外,如果 A
是一个包含整数 x
的开集,您只需 at x within A = at x
.
通常,如果您想要单边限制之类的东西(或者,在更高的维度中,如果您想以某种方式限制接近的方向),您只需要 has_field_derivative
和 at x within …
.
这是一个关于 Isabelle 库中导数概念的问题。
我正在尝试理解 (f has_field_derivative D x) (at x within S)
的含义。我知道 (at x within S)
是一个过滤器,但直觉上我在想下面的语句是真的
lemma DERIV_at_within:
"(∀x ∈ S. (f has_field_derivative D x) (at x))
= (∀x. (f has_field_derivative D x) (at x within S))"
如果不是,我还应该如何解释 (at x within S)
在导数的上下文中?
at x within A
是x
的尖邻域,与A
相交。例如,at_right
是at x within {x<..}
的缩写,即x
的右邻域。这允许您表达单边导数。
偶尔也会看到像∀x∈{a..b}. (f has_field_derivative f' x) (at x within {a..b})
这样的假设。这意味着 f
与导数 f'
在 a
和 b
之间是可微的,但是边缘处的导数(即在 a
和 b
) 只需要是单方面的。
另请注意 at x = at x within UNIV
。此外,如果 A
是一个包含整数 x
的开集,您只需 at x within A = at x
.
通常,如果您想要单边限制之类的东西(或者,在更高的维度中,如果您想以某种方式限制接近的方向),您只需要 has_field_derivative
和 at x within …
.