Skip to content

Commit

Permalink
Sets/GCHtoAC: simplify further
Browse files Browse the repository at this point in the history
  • Loading branch information
jdchristensen committed Sep 3, 2023
1 parent 33f9950 commit d4e3bd5
Showing 1 changed file with 2 additions and 3 deletions.
5 changes: 2 additions & 3 deletions theories/Sets/GCHtoAC.v
Original file line number Diff line number Diff line change
Expand Up @@ -68,9 +68,8 @@ Context {EM : ExcludedMiddle}.
Lemma PE (P P' : HProp) :
P <-> P' -> P = P'.
Proof.
intros [f g]. apply path_trunctype.
apply (equiv_adjointify f g).
all: intro x; apply path_ishprop.
intros iff. apply path_trunctype.
rapply (equiv_iff_hprop_uncurried iff).
Qed.

Lemma path_bool_prop :
Expand Down

0 comments on commit d4e3bd5

Please sign in to comment.