setquot is a set
authorAnders Mörtberg <andersmortberg@gmail.com>
Fri, 15 Jan 2016 03:55:34 +0000 (22:55 -0500)
committerAnders Mörtberg <andersmortberg@gmail.com>
Fri, 15 Jan 2016 03:55:34 +0000 (22:55 -0500)
examples/setquot.ctt

index ec2db10ea1619e3cd22d3fe7f76a4afabeacca44..0efaa96f5e8417fcbfc4ccf86353eda883e097d4 100644 (file)
@@ -183,17 +183,14 @@ setquotuniv2prop (X : U) (R : eqrel X) (P : setquot X R.1 -> setquot X R.1 -> hP
       (\ (x : X) -> setquotunivprop X R (\ (c0 : setquot X R.1) -> P c0 (setquotpr X R x))
                       (\ (x0 : X) -> ps x0 x) c) c'
 
-isincl (X Y : U) (f : X -> Y) : U = (y : Y) -> prop (fiber X Y f y)
-
-
--- Theorem isasetsetquot {X : UU} (R : hrel X) : isaset (setquot R).
--- Proof.
--- apply (isasetsubset (@pr1 _ _) (isasethsubtypes X)).
--- apply isinclpr1; intro x.
--- apply isapropiseqclass.
--- Defined.
+setsetquot (X : U) (R : hrel X) : set (setquot X R) =
+  setSig (hsubtypes X) (\(A : hsubtypes X) -> iseqclass X R A)
+    sA sB
+    where
+    sA : set (hsubtypes X) = sethsubtypes X
+    sB (x : hsubtypes X) : set (iseqclass X R x) = propSet (iseqclass X R x) (propiseqclass X R x)
 
-setsetquot (X : U) (R : hrel X) : set (setquot X R) = undefined
+isincl (X Y : U) (f : X -> Y) : U = (y : Y) -> prop (fiber X Y f y)
 
 iscompsetquotpr (X : U) (R : eqrel X) (x x' : X) (a : (R.1 x x').1) :
   Id (setquot X R.1) (setquotpr X R x) (setquotpr X R x') = undefined