- html - 出于某种原因,IE8 对我的 Sass 文件中继承的 html5 CSS 不友好?
- JMeter 在响应断言中使用 span 标签的问题
- html - 在 :hover and :active? 上具有不同效果的 CSS 动画
- html - 相对于居中的 html 内容固定的 CSS 重复背景?
以下两个命题很容易证明。
Theorem nat_eq_nat : nat = nat.
Proof.
trivial.
Qed.
Theorem True_neq_False : ~(True = False).
Proof.
unfold not.
intros.
symmetry in H.
rewrite H.
trivial.
Qed.
但是当我试图证明一个稍微不同的命题 ~(nat = False)
时,我发现重写策略不起作用。它报告
Error: Refiner was given an argument "fun x : Set => x" of type "Set -> Set" instead of "Set -> Prop".
所以我试着写一个引理。
Lemma Type_eq_prod : forall (a : Type) (b : Type), a = b -> (a -> b).
Proof.
intros.
rewrite <- H.
trivial.
Qed.
Theorem nat_neq_False : ~(nat = False).
Proof.
unfold not.
intros.
apply (Type_eq_prod nat False) in H.
inversion H.
apply 0. (*no subgoals left*)
到目前为止一切正常。但是当我尝试Qed它时,它报告了
Error: Illegal application (Type Error):
The term "Type_eq_prod" of type "forall a b : Type, a = b -> a -> b"
cannot be applied to the terms
"nat" : "Set"
"False" : "Prop"
"H" : "nat = False"
"0" : "nat"
The 3rd term has type "nat = False" which should be coercible to
"nat = False".
以下是另外两个让我卡住的命题。
Theorem nat_neq_bool : ~(nat = bool).
Proof.
unfold not.
intros.
Abort.
Theorem nat_neq_true : ~(nat = True).
Proof.
unfold not.
intros.
Abort.
我的问题是:
1.Why the rewrite tactic doesn't work with proposition ~(nat = False).
2.Why can't I Qed it when there is no subgoals.
3.How to prove the aborted propositions above or is it possible to prove or prove the negates of them in coq.
最佳答案
由于 Coq 处理其 Universe 的方式,重写策略不起作用,Prop
, Set
和 Type
.有一种包含的概念,它允许使用 Prop
好像它是一个 Set
或 Type
.这就是为什么你被允许写 nat = False
首先,因为平等只允许在相同类型的事物之间。问题在于,对于 Coq,False : Prop
不同于 False : Set
. not
用 False : Prop
定义,这意味着重写将产生不匹配,这解释了您收到的错误消息。
以下是可行的类似方法。注意对 Set
的显式强制.
Lemma nat_neq_False_2 : (nat = False) -> (False : Set).
Proof.
intros H.
rewrite <- H.
apply 0.
Qed.
Lemma nat_neq_False_3 : ~(nat = False).
Proof.
intros H.
destruct (nat_neq_False_2 H).
Qed.
当您使用策略编写证明时,Coq 本质上是在内部构建一个证明术语,但并没有真正对其进行类型检查。从这个意义上说,它有点像元编程。一旦你点击 Qed
,由策略构建的术语被发送到类型检查器以确保它是正确的。大多数时候,策略会产生正确的证明,但每隔一段时间就会发现不被接受的证明,您的案例就是一个例子。
打印的错误信息不是很清楚,但是可以通过使用命令 Set Printing All
更好地了解发生了什么。 ,这会导致 Coq 打印所有没有符号的术语和语句,并显示隐含的参数。这就是您的错误消息在执行此操作时的样子:
Set Printing All.
Lemma Type_eq_prod : forall (a : Type) (b : Type), a = b -> (a -> b).
Proof.
intros.
rewrite <- H.
trivial.
Qed.
Theorem nat_neq_False : ~(nat = False).
Proof.
unfold not.
intros.
apply (Type_eq_prod nat False) in H.
inversion H.
apply 0. (*no subgoals left*)
Qed.
(* Error: Illegal application (Type Error): *)
(* The term "Type_eq_prod" of type "forall a b : Type, @eq Type a b -> a -> b" *)
(* cannot be applied to the terms *)
(* "nat" : "Set" *)
(* "False" : "Prop" *)
(* "H" : "@eq Set nat False" *)
(* "O" : "nat" *)
(* The 3rd term has type "@eq Set nat False" which should be coercible to *)
(* "@eq Type nat False". *)
在那里,我们可以看到问题是再次出现了全域不匹配:Type
中存在一个相等性。 , 而另一个在 Set
.有几种方法可以解决这个问题;最简单的可能是将您的第一个定理更改为:
Lemma Type_eq_prod : forall (a : Set) (b : Set), a = b -> (a -> b).
这两个命题在 Coq 中都是可证明的。在 Coq 的基础理论中,唯一可以证明简单类型如 nat
和 bool
不同的是基数论点。因此,nat <> bool
因为bool
只有两个元素,而 nat
不止于此。因此,通过证明 bool
有两个元素,一个可以重写等式nat = bool
找出 nat
也应该有两个元素,然后利用它来得到一个矛盾。类似的论点将表明 nat <> True
.
关于functional-programming - 如何在 coq 中证明 "~(nat = False)"、 "~(nat = bool)"和 "~(nat = True)",我们在Stack Overflow上找到一个类似的问题: https://stackoverflow.com/questions/26550046/
main.cpp #include "Primes.h" #include int main(){ std::string choose; int num1, num2; w
似乎函数 qwertyInches() 应该可以工作但是当我在 main() 中调用它时它给了我 [Error] called object 'qwertyInches' is not a funct
我无法理解 C++ 语法的工作原理。 #include using namespace std; class Accumulator{ private: int value; public:
在 类中声明 函数成员时,我们可以同时执行这两种操作; Function first; Function() second; 它们之间有什么区别? 最佳答案 Function 代表任意函数: void
“colonna”怎么可能是一个简单的字符串: $('td.' + colonna).css('background-color','#ffddaa'); 可以正确突出显示有趣单元格的背景,并且: $
我正在尝试将网页中的动态参数中继到函数中,然后函数将它们传递给函数内部的调用。比如下面这个简化的代码片段,现在这样,直接传入参数是没有问题的。但是,如何在不为每个可能的 colorbox 参数设置 s
C++ 中是否有一种模式允许您返回一个函数,它返回一个函数本身。例如 std::function func = ...; do { func = func(); } while (func);
我正在将 Windows 程序集移植到 Linux。我有一些代码要移植。我实际上是 linux 中 C 的新手。我知道 C 基础知识是一样的! typedef struct sReader {
我一直在寻找一个很好的解释,所以我很清楚。示例: this.onDeleteHandler(index)}/> 对比 对比 this.nameChangedhandler(event, perso
function(){}.__proto__ === Function.prototype 和 Function.prototype === function(){}.__proto__ 得到不同的结
https://developer.mozilla.org/en-US/docs/Web/JavaScript/Reference/Global_Objects/Function 据说 Propert
VBA 中的函数没有特殊类型。我很难理解如何在 Excel VBA 中将函数作为参数添加到函数中。 我想要完成的是这样的事情: function f(g as function, x as strin
所以我正在尝试制作一个包(我没有在下面包含我的 roxygen2 header ): 我有这个功能: date_from_text % dplyr::mutate(!!name := lubr
尝试从 std::function 派生一个类,对于初学者来说,继承构造函数。这是我的猜测: #include #include using namespace std; template cla
我正在尝试编写一个返回另一个函数的函数。我的目标是编写一个函数,它接受一个对象并返回另一个函数“search”。当我使用键调用搜索函数时,我想从第一个函数中给定的对象返回该键的值。 propertyO
我非常清楚函数式编程技术和命令式编程技术之间的区别。但是现在有一种普遍的趋势是谈论“函数式语言”,这确实让我感到困惑。 当然,像 Haskell 这样的一些语言比 C 等其他语言更欢迎函数式编程。但即
关闭。这个问题是opinion-based 。目前不接受答案。 想要改进这个问题吗?更新问题,以便 editing this post 可以用事实和引文来回答它。 . 已关闭 8 年前。 Improv
我在stackoverflow上查过很多类似的问题,比如call.call 1 , call.call 2 ,但我是新人,无法发表任何评论。我希望我能找到关于 JavaScript 解释器如何执行这些
向 Twilio 发送 SMS 时,Twilio 会向指定的 URL 发送多个请求,以通过 Webhook 提供该 SMS 传送的状态。我想让这个回调异步,所以我开发了一个 Cloud Functio
作为 IaC 的一部分,A 功能应用 ,让我们将其命名为 FuncAppX 是使用 Terraform 部署的,它有一个内置函数。 我需要使用 Terraform 在函数应用程序中访问相同函数的 Ur
我是一名优秀的程序员,十分优秀!