2015-04-10 01:45:18 +00:00
|
|
|
/-
|
|
|
|
Copyright (c) 2015 Floris van Doorn. All rights reserved.
|
|
|
|
Released under Apache 2.0 license as described in the file LICENSE.
|
|
|
|
Authors: Floris van Doorn
|
|
|
|
|
|
|
|
Declaration of set-quotients
|
|
|
|
-/
|
|
|
|
|
2015-04-11 00:33:33 +00:00
|
|
|
import .type_quotient .trunc
|
2015-04-10 01:45:18 +00:00
|
|
|
|
2015-04-11 00:33:33 +00:00
|
|
|
open eq is_trunc trunc type_quotient
|
2015-04-10 01:45:18 +00:00
|
|
|
|
|
|
|
namespace quotient
|
2015-04-23 22:27:56 +00:00
|
|
|
section
|
2015-04-11 00:33:33 +00:00
|
|
|
parameters {A : Type} (R : A → A → hprop)
|
|
|
|
-- set-quotients are just truncations of type-quotients
|
|
|
|
definition quotient : Type := trunc 0 (type_quotient (λa a', trunctype.carrier (R a a')))
|
2015-04-10 01:45:18 +00:00
|
|
|
|
|
|
|
definition class_of (a : A) : quotient :=
|
2015-04-11 00:33:33 +00:00
|
|
|
tr (class_of _ a)
|
2015-04-10 01:45:18 +00:00
|
|
|
|
|
|
|
definition eq_of_rel {a a' : A} (H : R a a') : class_of a = class_of a' :=
|
2015-04-27 21:34:55 +00:00
|
|
|
ap tr (eq_of_rel _ H)
|
2015-04-10 01:45:18 +00:00
|
|
|
|
2015-04-11 00:33:33 +00:00
|
|
|
theorem is_hset_quotient : is_hset quotient :=
|
2015-04-25 00:21:08 +00:00
|
|
|
begin unfold quotient, exact _ end
|
2015-04-10 01:45:18 +00:00
|
|
|
|
2015-04-19 21:56:24 +00:00
|
|
|
protected definition rec {P : quotient → Type} [Pt : Πaa, is_hset (P aa)]
|
2015-05-01 03:23:12 +00:00
|
|
|
(Pc : Π(a : A), P (class_of a)) (Pp : Π⦃a a' : A⦄ (H : R a a'), eq_of_rel H ▸ Pc a = Pc a')
|
2015-04-10 01:45:18 +00:00
|
|
|
(x : quotient) : P x :=
|
|
|
|
begin
|
|
|
|
apply (@trunc.rec_on _ _ P x),
|
|
|
|
{ intro x', apply Pt},
|
2015-04-11 00:33:33 +00:00
|
|
|
{ intro y, fapply (type_quotient.rec_on y),
|
2015-04-10 01:45:18 +00:00
|
|
|
{ exact Pc},
|
2015-05-03 05:22:31 +00:00
|
|
|
{ intros,
|
|
|
|
apply concat, apply transport_compose; apply Pp}}
|
2015-04-10 01:45:18 +00:00
|
|
|
end
|
|
|
|
|
|
|
|
protected definition rec_on [reducible] {P : quotient → Type} (x : quotient)
|
2015-04-19 21:56:24 +00:00
|
|
|
[Pt : Πaa, is_hset (P aa)] (Pc : Π(a : A), P (class_of a))
|
2015-05-01 03:23:12 +00:00
|
|
|
(Pp : Π⦃a a' : A⦄ (H : R a a'), eq_of_rel H ▸ Pc a = Pc a') : P x :=
|
2015-04-10 01:45:18 +00:00
|
|
|
rec Pc Pp x
|
|
|
|
|
2015-04-27 21:34:55 +00:00
|
|
|
theorem rec_eq_of_rel {P : quotient → Type} [Pt : Πaa, is_hset (P aa)]
|
2015-05-01 03:23:12 +00:00
|
|
|
(Pc : Π(a : A), P (class_of a)) (Pp : Π⦃a a' : A⦄ (H : R a a'), eq_of_rel H ▸ Pc a = Pc a')
|
2015-04-27 21:34:55 +00:00
|
|
|
{a a' : A} (H : R a a') : apd (rec Pc Pp) (eq_of_rel H) = Pp H :=
|
2015-04-28 01:30:20 +00:00
|
|
|
!is_hset.elim
|
2015-04-10 01:45:18 +00:00
|
|
|
|
2015-04-19 21:56:24 +00:00
|
|
|
protected definition elim {P : Type} [Pt : is_hset P] (Pc : A → P)
|
2015-04-10 01:45:18 +00:00
|
|
|
(Pp : Π⦃a a' : A⦄ (H : R a a'), Pc a = Pc a') (x : quotient) : P :=
|
|
|
|
rec Pc (λa a' H, !tr_constant ⬝ Pp H) x
|
|
|
|
|
2015-04-19 21:56:24 +00:00
|
|
|
protected definition elim_on [reducible] {P : Type} (x : quotient) [Pt : is_hset P]
|
2015-04-10 01:45:18 +00:00
|
|
|
(Pc : A → P) (Pp : Π⦃a a' : A⦄ (H : R a a'), Pc a = Pc a') : P :=
|
|
|
|
elim Pc Pp x
|
|
|
|
|
2015-04-27 21:34:55 +00:00
|
|
|
theorem elim_eq_of_rel {P : Type} [Pt : is_hset P] (Pc : A → P)
|
2015-04-10 01:45:18 +00:00
|
|
|
(Pp : Π⦃a a' : A⦄ (H : R a a'), Pc a = Pc a') {a a' : A} (H : R a a')
|
2015-04-27 21:34:55 +00:00
|
|
|
: ap (elim Pc Pp) (eq_of_rel H) = Pp H :=
|
|
|
|
begin
|
|
|
|
apply (@cancel_left _ _ _ _ (tr_constant (eq_of_rel H) (elim Pc Pp (class_of a)))),
|
|
|
|
rewrite [-apd_eq_tr_constant_con_ap,↑elim,rec_eq_of_rel],
|
|
|
|
end
|
|
|
|
|
|
|
|
/-
|
|
|
|
there are no theorems to eliminate to the universe here,
|
|
|
|
because the universe is generally not a set
|
|
|
|
-/
|
2015-04-10 01:45:18 +00:00
|
|
|
|
|
|
|
end
|
|
|
|
end quotient
|
2015-05-07 20:35:14 +00:00
|
|
|
|
|
|
|
attribute quotient.class_of [constructor]
|
|
|
|
attribute quotient.rec quotient.elim [unfold-c 7]
|
|
|
|
attribute quotient.rec_on quotient.elim_on [unfold-c 4]
|