File: HoTT_coq_059.v

package info (click to toggle)
coq 8.20.1%2Bdfsg-1
  • links: PTS, VCS
  • area: main
  • in suites: sid, trixie
  • size: 44,116 kB
  • sloc: ml: 234,160; sh: 4,301; python: 3,270; ansic: 2,644; makefile: 882; lisp: 172; javascript: 63; xml: 24; sed: 2
file content (18 lines) | stat: -rw-r--r-- 672 bytes parent folder | download | duplicates (2)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
(* -*- mode: coq; coq-prog-args: ("-indices-matter") -*- *)
Set Universe Polymorphism.

Inductive eq {A} (x : A) : A -> Type := eq_refl : eq x x.
Notation "a = b" := (eq a b) : type_scope.

Section foo.
  Class Funext := { path_forall :: forall A P (f g : forall x : A, P x), (forall x, f x = g x) -> f = g }.
  Context `{Funext, Funext}.

  Set Printing Universes.

  (** Typeclass resolution should pick up the different instances of Funext automatically *)
  Definition foo := (@path_forall _ _ _ (@path_forall _ Set)).
  (* Toplevel input, characters 0-60:
Error: Universe inconsistency (cannot enforce Top.24 <= Top.23 because Top.23
< Top.22 <= Top.24). *)
End foo.