关于一些伸张平等公理的相对强弱

时间:2018-01-14 12:06:35

标签: coq

鉴于以下公理:

Definition Axiom1 : Prop := forall (a b:Type) (f g: a -> b),
    (forall x, f x = g x) -> f = g.


Definition Axiom2 : Prop := forall (a:Type) (B:a -> Type) (f g: forall x, B x),
    (forall x, f x = g x) -> f = g.

可以很容易地证明Axiom2Axiom1更强大的公理:

Theorem Axiom2ImpAxiom1 : Axiom2 -> Axiom1.
Proof.
    intros H a b f g H'. apply H. exact H'.
Qed.

有没有人知道(在Coq的类型理论中),这两个公理实际上是等价的,还是已知它们不是。如果相同,是否有一个简单的Coq证明事实?

1 个答案:

答案 0 :(得分:2)

是的,这两个公理是等价的;关键是要经过fun x => existT B x (f x)fun x => existT B x (g x),尽管必须要做一些棘手的平等推理。在https://github.com/HoTT/HoTT/blob/c54a967526bb6293a0802cb2bed32e0b4dbe5cdc/contrib/old/Funext.v#L113-L358处有一个几乎完整的证明,其使用的术语略有不同。