-
Notifications
You must be signed in to change notification settings - Fork 0
/
Copy pathHoTT_coq_102.v
30 lines (24 loc) · 1.01 KB
/
HoTT_coq_102.v
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
22
23
24
25
26
27
28
29
30
Require Import TestSuite.admit.
(* File reduced by coq-bug-finder from 64 lines to 30 lines. *)
Set Implicit Arguments.
Set Universe Polymorphism.
Generalizable All Variables.
Record SpecializedCategory (obj : Type) := { Object :> _ := obj }.
Record > Category :=
{ CObject : Type;
UnderlyingCategory :> @SpecializedCategory CObject }.
Record SpecializedFunctor `(C : @SpecializedCategory objC) `(D : @SpecializedCategory objD) :=
{ ObjectOf :> objC -> objD }.
Definition Functor (C D : Category) := SpecializedFunctor C D.
Parameter TerminalCategory : SpecializedCategory unit.
Definition focus A (_ : A) := True.
Definition CommaCategory_Object (A : Category) (S : Functor TerminalCategory A) : Type.
assert (Hf : focus ((S tt) = (S tt))) by constructor.
let C1 := constr:(CObject) in
let C2 := constr:(fun C => @Object (CObject C) C) in
let check := constr:(eq_refl : C1 = C2) in
unify C1 C2.
progress change CObject with (fun C => @Object (CObject C) C) in *.
(* not convertible *)
admit.
Defined.