英文: Replace element in Coq list 问题 I am writing Coq code that needs to modify lists, particularly by...
Coerce rat to realType im math-comp/analysis
英文: Coerce rat to realType im math-comp/analysis 问题 There is a way to coerce a rat into a realType u...
“接受任意数量量词的Ltac策略”
英文: Ltac tactic that accepts an arbitrary number of quantifiers 问题 I'm trying to write a--my first--...
Syntax error: '.' expected after [vernac:gallina] (in [vernac_aux]) in Coq when using inductive with integers
英文: Syntax error: '.' expected after [vernac:gallina] (in [vernac_aux]) in Coq when using in...
有没有在Coq中可以处理布尔值的集合库?
英文: Is there a library for sets that works with bool in Coq? 问题 我正在寻求使用数学集合和某种通用类型的子集进行工作。 我知道通常这表示为...
Morphism signature for dependently-typed vectors in Coq
英文: Morphism signature for dependently-typed vectors in coq 问题 I want to be able to rewrite terms in...
Fail to `destruct` due to ill-typedness and even cannot give an exact term in Coq
英文: Fail to `destruct` due to ill-typedness and even cannot give an exact term in Coq 问题 以下是您要翻译的内容:...
如何确保Coq项目安装正确,当它似乎不出现在opam列表中?
英文: How does one make sure that coq project installed correctly when it doesn't seem to appear o...
“Does `∃! x, ∃! y, P (x, y)` imply `∃! xy, P (fst xy) (snd xy)`?”
英文: Does `∃! x, ∃! y, P (x, y)` imply `∃! xy, P (fst xy) (snd xy)`? 问题 以下是翻译好的部分: 可以相对容易地证明以下内容(Coq)...
如何仅扩展 `fix` 函数一步?
英文: How does one expand a `fix` function just one step? 问题 I have defined a recursive function with ...
3