Skip to content
Snippets Groups Projects
Commit 835d3d76 authored by Gregory Malecha's avatar Gregory Malecha Committed by Gregory Malecha
Browse files

Use unicode and fix comment.

parent a0d4deb1
No related branches found
No related tags found
1 merge request!368Define [tele_arg] as a fixpoint
...@@ -48,6 +48,7 @@ is essentially just a (dependent) product. ...@@ -48,6 +48,7 @@ is essentially just a (dependent) product.
*) *)
Definition no_bump@{u} (t : tele@{u}) : Type@{u} := tele_arg@{u} t. Definition no_bump@{u} (t : tele@{u}) : Type@{u} := tele_arg@{u} t.
Lemma texist_exist_universes (X : Type) (P : TeleS (fun _ : X => TeleO) -> Prop) : (** This test would fail without [Unset Universe Minimization ToSet] in [telescopes.v]. *)
texist P <-> ex P. Lemma texist_exist_universes (X : Type) (P : TeleS (λ _ : X, TeleO) Prop) :
texist P ex P.
Proof. by rewrite texist_exist. Qed. Proof. by rewrite texist_exist. Qed.
...@@ -3,8 +3,9 @@ From stdpp Require Import options. ...@@ -3,8 +3,9 @@ From stdpp Require Import options.
Local Set Universe Polymorphism. Local Set Universe Polymorphism.
(* Without this flag, Coq minimizes some universes to [Set] when they (** Without this flag, Coq minimizes some universes to [Set] when they
should not be, e.g. in [texist_exist]. *) should not be, e.g. in [texist_exist].
See the [texist_exist_universes] test. *)
Local Unset Universe Minimization ToSet. Local Unset Universe Minimization ToSet.
(** Telescopes *) (** Telescopes *)
...@@ -75,7 +76,7 @@ Lemma tele_arg_inv {TT : tele} (a : tele_arg TT) : ...@@ -75,7 +76,7 @@ Lemma tele_arg_inv {TT : tele} (a : tele_arg TT) :
| TeleS f => λ a, x a', a = TargS x a' | TeleS f => λ a, x a', a = TargS x a'
end a. end a.
Proof. destruct TT; destruct a; eauto. Qed. Proof. destruct TT; destruct a; eauto. Qed.
Lemma tele_arg_O_inv (a : TeleO) : a = (). Lemma tele_arg_O_inv (a : TeleO) : a = TargO.
Proof. exact (tele_arg_inv a). Qed. Proof. exact (tele_arg_inv a). Qed.
Lemma tele_arg_S_inv {X} {f : X tele} (a : TeleS f) : Lemma tele_arg_S_inv {X} {f : X tele} (a : TeleS f) :
x a', a = TargS x a'. x a', a = TargS x a'.
......
0% Loading or .
You are about to add 0 people to the discussion. Proceed with caution.
Finish editing this message first!
Please register or to comment