Skip to content

Commit

Permalink
feat(topology/instances/ereal): more on ereal, notably its topology (#…
Browse files Browse the repository at this point in the history
  • Loading branch information
sgouezel committed Jun 8, 2021
1 parent 75c81de commit 5c6d3bc
Show file tree
Hide file tree
Showing 4 changed files with 723 additions and 21 deletions.
4 changes: 4 additions & 0 deletions src/algebra/ordered_monoid.lean
Expand Up @@ -464,6 +464,10 @@ begin
exact ⟨_, rfl, add_le_add_left h _⟩, }
end

instance [linear_ordered_add_comm_monoid α] : linear_ordered_add_comm_monoid (with_bot α) :=
{ ..with_bot.linear_order,
..with_bot.ordered_add_comm_monoid }

-- `by norm_cast` proves this lemma, so I did not tag it with `norm_cast`
lemma coe_zero [has_zero α] : ((0 : α) : with_bot α) = 0 := rfl

Expand Down

0 comments on commit 5c6d3bc

Please sign in to comment.