考虑以下语言环境定义:
locale my_locale =
fixes a :: nat
assumes "a > 0"
begin
definition "f n ≡ a + n"
lemma f_pos: "f x > 0"
sorry
end
在Isar中,如果我尝试使用f
或引理f_pos
的定义,那么区域设置假设和固定变量对我来说是隐藏的。例如,thm f_def f_pos
返回:
f ?n ≡ a + ?n
0 < f ?x
正如所料。
但是,如果我试图在ML中推理这些术语,那么“隐藏的”固定变量会突然暴露出来。例如,ML {* @{thm f_def} |> prop_of *}
返回:
Const ("==", "nat ⇒ nat ⇒ prop") $
(Const ("TestSimple.my_locale.f", "nat ⇒ nat ⇒ nat") $
Free ("a", "nat") $ Var (("n", 0), "nat")) $
(Const ("Groups.plus_class.plus", "nat ⇒ nat ⇒ nat") $
Free ("a", "nat") $ Var (("n", 0), "nat"))
其中固定变量a
成为函数f
的参数。
有没有办法在ML中的语言环境中工作,这样我就不会接触到这样的语言环境变量?
答案 0 :(得分:1)
似乎f
的版本没有参数a
,只是locale
命令生成的缩写。特别是,键入print_abbrevs
会显示:
local.f ≡ My_Theory.my_locale.f a
这意味着从用户的角度来看,f
似乎没有任何区域设置参数,因为它们隐藏在缩写后面。但是,在幕后,f
将始终附加locale参数,因此必须对ML代码进行编码以显式处理它。