Skip to content

Commit

Permalink
docs(data/fp): Move title comment so that it appears in the markdown (#…
Browse files Browse the repository at this point in the history
  • Loading branch information
eric-wieser committed Dec 4, 2020
1 parent 30467f4 commit 54c13bd
Showing 1 changed file with 3 additions and 2 deletions.
5 changes: 3 additions & 2 deletions src/data/fp/basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -2,11 +2,12 @@
Copyright (c) 2017 Mario Carneiro. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Mario Carneiro
Implementation of floating-point numbers (experimental).
-/
import data.rat
import data.semiquot
/-!
# Implementation of floating-point numbers (experimental).
-/

def int.shift2 (a b : ℕ) : ℤ → ℕ × ℕ
| (int.of_nat e) := (a.shiftl e, b)
Expand Down

0 comments on commit 54c13bd

Please sign in to comment.