什么是==&燃气轮机&引用;你的意思是coq?

什么是==&燃气轮机&引用;你的意思是coq?,coq,Coq,我有以下代码: 以下是分类的定义: Fixpoint sorted (l : list nat) := match l with | [] => true | x::xs => match xs with | [] => true | y :: ys => (x <=? y) && (sorted xs) end end. 在insert_s

我有以下代码: 以下是分类的定义:

Fixpoint sorted (l : list nat) := 
  match l with 
  | [] => true 
  | x::xs => match xs with 
             | [] => true 
             | y :: ys => (x <=? y) && (sorted xs) 
             end 
  end.

在insert_spec中,“==>”是什么意思?

您似乎是从软件基金会获得代码的。该指南中使用的许多(如果不是全部)符号可在中找到。在这里,我们发现
“==>”
被定义为一种符号

Module QcNotation.
  Export QcDefaultNotation.
  Notation "x ==> y" :=
    (implication x y) (at level 55, right associativity)
    : Checker_scope.
End QcNotation.
implication
是QuickChick使用的通用“Isthis implication true”参数

Parameter implication :
  ∀ {prop : Type} `{Checkable prop} (b : bool) (p : prop), Checker.
每当第一个参数为true时,QuickChick都会测试第二个参数的计算结果(在您使用QuickChick的任何上下文中)是否也为true


因此,对于您的特定代码,
“==>”
用于表示我们希望测试,无论何时对
l
进行排序,
insert x l
也会进行排序。

您似乎从软件基础获得了代码。该指南中使用的许多(如果不是全部)符号可在中找到。在这里,我们发现
“==>”
被定义为一种符号

Module QcNotation.
  Export QcDefaultNotation.
  Notation "x ==> y" :=
    (implication x y) (at level 55, right associativity)
    : Checker_scope.
End QcNotation.
implication
是QuickChick使用的通用“Isthis implication true”参数

Parameter implication :
  ∀ {prop : Type} `{Checkable prop} (b : bool) (p : prop), Checker.
每当第一个参数为true时,QuickChick都会测试第二个参数的计算结果(在您使用QuickChick的任何上下文中)是否也为true


因此,对于您的特定代码,
“==>”
用于表示我们希望测试,每当对
l
进行排序时,
insert x l
也会进行排序。

这不是标准的表示法。知道你从哪里得到的代码会有帮助。这不是一个标准的符号。知道你从哪里得到这个密码会有帮助。