Coq Ltac:根据包含用户定义符号的假设与Ltac匹配

Coq Ltac:根据包含用户定义符号的假设与Ltac匹配,coq,coq-tactic,ltac,Coq,Coq Tactic,Ltac,我对ordType有以下定义,对其布尔比较运算符有中缀符号=,这是因为强制是真的--H假设实际上是H:is\u真的(x==y) 如果启用如下方式打印强制,则可以看到: Set Printing Coercions. 有些库实现了ordType,例如。 Ltac show_H:= match goal with | H: ?x == ?y |- _ => idtac H end. Lemma triv (T:ordType)(x y:T): x == y -> y &

我对
ordType
有以下定义,对其布尔比较运算符有中缀符号
=
这是因为强制
是真的--
H
假设实际上是
H:is\u真的(x==y)

如果启用如下方式打印强制,则可以看到:

Set Printing Coercions.

有些库实现了
ordType
,例如。
Ltac show_H:=
  match goal with
  | H: ?x == ?y |- _ =>  idtac H
 end.
 Lemma triv (T:ordType)(x y:T): x == y -> y <b x -> 2=3.
 Proof. intros. show_H. 

 (Error: No matching clauses for match)
Set Printing Coercions.