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 @@ -1375,12 +1375,9 @@ Proof.
13751375 apply subtypePath; simpl.
13761376 intros x; apply isapropdirprod; apply setproperty.
13771377 refine (@toforallpaths unitset _ (fun _ => ab) (fun _ => ab') _ tt).
1378- admit.
1379- (*
1380- use (MorphismsIntoPullbackEqual);
1378+ refine (MorphismsIntoPullbackEqual pb _ _ _ _ _ );
13811379 apply funextsec; intros []; cbn;
13821380 (eapply @pathscomp0; [ eassumption | apply pathsinv0; eassumption]).
1383- *)
13841381 - simple refine (_,,_).
13851382 refine (_ tt).
13861383 refine (PullbackArrow Pb (unitset : HSET)
@@ -1391,7 +1388,7 @@ Proof.
13911388 apply (PullbackArrow_PullbackPr1 Pb unitset).
13921389 + generalize tt; apply toforallpaths.
13931390 apply (PullbackArrow_PullbackPr2 Pb unitset).
1394- Admitted .
1391+ Defined .
13951392
13961393Lemma pullback_HSET_elements_unique {P A B C : HSET}
13971394 {p1 : HSET ⟦ P, A ⟧} {p2 : HSET ⟦ P, B ⟧}
You can’t perform that action at this time.
0 commit comments