Skip to content

Commit dd2ca5c

Browse files
authored
Merge pull request #2252 from jdchristensen/export-instances
EMSpace: add #[export] to the instances
2 parents feea9f2 + 28d1ed7 commit dd2ca5c

File tree

1 file changed

+4
-4
lines changed

1 file changed

+4
-4
lines changed

theories/Homotopy/EMSpace.v

+4-4
Original file line numberDiff line numberDiff line change
@@ -29,27 +29,27 @@ Notation "'K(' G , n )" := (EilenbergMacLane G n).
2929
Section EilenbergMacLane.
3030
Context `{Univalence}.
3131

32-
Instance istrunc_em {G : Group} {n : nat} : IsTrunc n K(G, n).
32+
#[export] Instance istrunc_em {G : Group} {n : nat} : IsTrunc n K(G, n).
3333
Proof.
3434
destruct n as [|[]]; exact _.
3535
Defined.
3636

3737
(** This is subsumed by the next result, but Coq doesn't always find the next result when it should. *)
38-
Instance isconnected_em {G : Group} (n : nat)
38+
#[export] Instance isconnected_em {G : Group} (n : nat)
3939
: IsConnected n K(G, n.+1).
4040
Proof.
4141
induction n; exact _.
4242
Defined.
4343

44-
Instance isconnected_em' {G : Group} (n : nat)
44+
#[export] Instance isconnected_em' {G : Group} (n : nat)
4545
: IsConnected n.-1 K(G, n).
4646
Proof.
4747
destruct n.
4848
1: exact (is_minus_one_connected_pointed _).
4949
apply isconnected_em.
5050
Defined.
5151

52-
Instance is0connected_em {G : Group} (n : nat)
52+
#[export] Instance is0connected_em {G : Group} (n : nat)
5353
: IsConnected 0 K(G, n.+1).
5454
Proof.
5555
rapply (is0connected_isconnected n.-2).

0 commit comments

Comments
 (0)