Built with Alectryon, running Coq+SerAPI v8.19.0+0.19.3. Bubbles () indicate interactive fragments: hover for details, tap to reveal contents. Use Ctrl+↑Ctrl+↓ to navigate, Ctrl+🖱️ to focus. On Mac, use ⌘ instead of Ctrl.
[Loading ML file number_string_notation_plugin.cmxs (using legacy method) ... done]
Require Import Modality Accessible.LocalOpen Scope path_scope.(** * The identity modality *)(** Everything to say here is fairly trivial. *)
Modality
Modality
forallTU : Type,
(fun_ : Type => Unit) T ->
forallf : T -> U,
IsEquiv f -> (fun_ : Type => Unit) U
forallT : Type, (fun_ : Type => Unit) (idmap T)
forallT : Type, T -> idmap T
forall (A : Type) (B : idmap A -> Type),
(foralloa : idmap A, (fun_ : Type => Unit) (B oa)) ->
(foralla : A, B (?to' A a)) ->
forallz : idmap A, B z
forall (A : Type) (B : idmap A -> Type)
(B_inO : foralloa : idmap A,
(fun_ : Type => Unit) (B oa))
(f : foralla : A, B (?to' A a)) (a : A),
?O_ind' A B B_inO f (?to' A a) = f a
forallA : Type,
(fun_ : Type => Unit) A ->
forallzz' : A, (fun_ : Type => Unit) (z = z')
forallT : Type, T -> idmap T
forall (A : Type) (B : idmap A -> Type),
(foralloa : idmap A, (fun_ : Type => Unit) (B oa)) ->
(foralla : A, B (?to' A a)) ->
forallz : idmap A, B z
forall (A : Type) (B : idmap A -> Type)
(B_inO : foralloa : idmap A,
(fun_ : Type => Unit) (B oa))
(f : foralla : A, B (?to' A a)) (a : A),
?O_ind' A B B_inO f (?to' A a) = f a
forallT : Type, T -> idmap T
intros; assumption.
forall (A : Type) (B : idmap A -> Type),
(foralloa : idmap A, (fun_ : Type => Unit) (B oa)) ->
(foralla : A, B ((funT : Type => idmap) A a)) ->
forallz : idmap A, B z
intros ? ? ? f z; exact (f z).
forall (A : Type) (B : idmap A -> Type)
(B_inO : foralloa : idmap A,
(fun_ : Type => Unit) (B oa))
(f : foralla : A, B ((funT : Type => idmap) A a))
(a : A),
(fun (A0 : Type) (B0 : idmap A0 -> Type)
(_ : foralloa : idmap A0,
(fun_ : Type => Unit) (B0 oa))
(f0 : foralla0 : A0,
B0 ((funT : Type => idmap) A0 a0))
(z : idmap A0) => f0 z) A B B_inO f
((funT : Type => idmap) A a) = f a
intros; reflexivity.Defined.
IsAccModality purely
IsAccModality purely
NullGenerators
forallX : Type,
In purely X <-> IsNull_Internal.IsNull ?acc_ngen X
NullGenerators
?ngen_indices -> Type
exact (@Empty_rec Type).
forallX : Type,
In purely X <->
IsNull_Internal.IsNull
{| ngen_indices := Empty; ngen_type := Empty_rec |}
X
X: Type
In purely X ->
IsNull_Internal.IsNull
{| ngen_indices := Empty; ngen_type := Empty_rec |}
X
X: Type
IsNull_Internal.IsNull
{| ngen_indices := Empty; ngen_type := Empty_rec |}
X -> In purely X
X: Type
In purely X ->
IsNull_Internal.IsNull
{| ngen_indices := Empty; ngen_type := Empty_rec |}
X
intros _ [].
X: Type
IsNull_Internal.IsNull
{| ngen_indices := Empty; ngen_type := Empty_rec |}
X -> In purely X