File tree Expand file tree Collapse file tree 1 file changed +2
-5
lines changed
Expand file tree Collapse file tree 1 file changed +2
-5
lines changed Original file line number Diff line number Diff line change @@ -1393,12 +1393,9 @@ Proof.
13931393 apply subtypePath; simpl.
13941394 intros x; apply isapropdirprod; apply setproperty.
13951395 refine (@toforallpaths unitset _ (fun _ => ab) (fun _ => ab') _ tt).
1396- admit.
1397- (*
1398- use (MorphismsIntoPullbackEqual);
1396+ refine (MorphismsIntoPullbackEqual pb _ _ _ _ _ );
13991397 apply funextsec; intros []; cbn;
14001398 (eapply @pathscomp0; [ eassumption | apply pathsinv0; eassumption]).
1401- *)
14021399 - simple refine (_,,_).
14031400 refine (_ tt).
14041401 refine (PullbackArrow Pb (unitset : HSET)
@@ -1409,7 +1406,7 @@ Proof.
14091406 apply (PullbackArrow_PullbackPr1 Pb unitset).
14101407 + generalize tt; apply toforallpaths.
14111408 apply (PullbackArrow_PullbackPr2 Pb unitset).
1412- Admitted .
1409+ Defined .
14131410
14141411Lemma pullback_HSET_elements_unique {P A B C : HSET}
14151412 {p1 : HSET ⟦ P, A ⟧} {p2 : HSET ⟦ P, B ⟧}
You can’t perform that action at this time.
0 commit comments