aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/HoTT_coq_098.v
diff options
context:
space:
mode:
authorGravatar Jason Gross <jgross@mit.edu>2014-05-09 10:13:32 -0400
committerGravatar Matthieu Sozeau <mattam@mattam.org>2014-05-10 15:39:39 +0200
commitc7284415e4bdd3315c84c7d15d140d3fee000bc5 (patch)
treecc8ded3feba7e1da0dd4f7d17b7e5f974de752c3 /test-suite/bugs/closed/HoTT_coq_098.v
parent3f64bd23a343bcd7be0ef07afa7d9e3249df24ec (diff)
Move opened bugs to bugs/opened
Diffstat (limited to 'test-suite/bugs/closed/HoTT_coq_098.v')
-rw-r--r--test-suite/bugs/closed/HoTT_coq_098.v84
1 files changed, 0 insertions, 84 deletions
diff --git a/test-suite/bugs/closed/HoTT_coq_098.v b/test-suite/bugs/closed/HoTT_coq_098.v
deleted file mode 100644
index 1e7be20d5..000000000
--- a/test-suite/bugs/closed/HoTT_coq_098.v
+++ /dev/null
@@ -1,84 +0,0 @@
-Set Implicit Arguments.
-Generalizable All Variables.
-
-Polymorphic Record SpecializedCategory (obj : Type) := Build_SpecializedCategory' {
- Object :> _ := obj;
- Morphism' : obj -> obj -> Type;
-
- Identity' : forall o, Morphism' o o;
- Compose' : forall s d d', Morphism' d d' -> Morphism' s d -> Morphism' s d'
-}.
-
-Polymorphic Definition TypeCat : @SpecializedCategory Type
- := (@Build_SpecializedCategory' Type
- (fun s d => s -> d)
- (fun _ => (fun x => x))
- (fun _ _ _ f g => (fun x => f (g x)))).
-
-Inductive GraphIndex := GraphIndexSource | GraphIndexTarget.
-Polymorphic Definition GraphIndexingCategory : @SpecializedCategory GraphIndex.
-Admitted.
-
-Module success.
- Section SpecializedFunctor.
- Set Universe Polymorphism.
- Context `(C : @SpecializedCategory objC).
- Context `(D : @SpecializedCategory objD).
- Unset Universe Polymorphism.
-
- Polymorphic Record SpecializedFunctor
- := {
- ObjectOf' : objC -> objD;
- MorphismOf' : forall s d, C.(Morphism') s d -> D.(Morphism') (ObjectOf' s) (ObjectOf' d)
- }.
- End SpecializedFunctor.
-
- Polymorphic Definition UnderlyingGraph : SpecializedFunctor GraphIndexingCategory TypeCat.
- Admitted.
-End success.
-
-Module failure.
- Section SpecializedFunctor.
- Context `(C : @SpecializedCategory objC).
- Context `(D : @SpecializedCategory objD).
-
- Polymorphic Record SpecializedFunctor
- := {
- ObjectOf' : objC -> objD;
- MorphismOf' : forall s d, C.(Morphism') s d -> D.(Morphism') (ObjectOf' s) (ObjectOf' d)
- }.
- End SpecializedFunctor.
-
- Set Printing Universes.
- Fail Polymorphic Definition UnderlyingGraph : SpecializedFunctor GraphIndexingCategory TypeCat.
- (* Toplevel input, characters 73-94:
-Error:
-The term "GraphIndexingCategory (* Top.563 *)" has type
- "SpecializedCategory (* Top.563 Set *) GraphIndex"
-while it is expected to have type
- "SpecializedCategory (* Top.550 Top.551 *) ?7"
-(Universe inconsistency: Cannot enforce Set = Top.551)). *)
-End failure.
-
-Module polycontext.
- Section SpecializedFunctor.
- Polymorphic Context `(C : @SpecializedCategory objC).
- Polymorphic Context `(D : @SpecializedCategory objD).
-
- Polymorphic Record SpecializedFunctor
- := {
- ObjectOf' : objC -> objD;
- MorphismOf' : forall s d, C.(Morphism') s d -> D.(Morphism') (ObjectOf' s) (ObjectOf' d)
- }.
- End SpecializedFunctor.
-
- Set Printing Universes.
- Fail Polymorphic Definition UnderlyingGraph : SpecializedFunctor GraphIndexingCategory TypeCat.
- (* Toplevel input, characters 73-94:
-Error:
-The term "GraphIndexingCategory (* Top.563 *)" has type
- "SpecializedCategory (* Top.563 Set *) GraphIndex"
-while it is expected to have type
- "SpecializedCategory (* Top.550 Top.551 *) ?7"
-(Universe inconsistency: Cannot enforce Set = Top.551)). *)
-End polycontext.