Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit 300b765

Browse files
committed
fix(topology/order): Missing Prop annotation
1 parent e4fc5af commit 300b765

File tree

1 file changed

+1
-1
lines changed

1 file changed

+1
-1
lines changed

src/topology/order.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -125,7 +125,7 @@ lemma generate_from_mono {α} {g₁ g₂ : set (set α)} (h : g₁ ⊆ g₂) :
125125
instance {α : Type u} : complete_lattice (topological_space α) :=
126126
(gi_generate_from α).lift_complete_lattice
127127

128-
class discrete_topology (α : Type*) [t : topological_space α] :=
128+
class discrete_topology (α : Type*) [t : topological_space α] : Prop :=
129129
(eq_top : t = ⊤)
130130

131131
@[simp] lemma is_open_discrete [topological_space α] [discrete_topology α] (s : set α) :

0 commit comments

Comments
 (0)