File tree Expand file tree Collapse file tree 4 files changed +11
-3
lines changed Expand file tree Collapse file tree 4 files changed +11
-3
lines changed Original file line number Diff line number Diff line change @@ -20,6 +20,8 @@ We define many of the bitvector operations from the
20
20
of SMT-LIBv2.
21
21
-/
22
22
23
+ set_option linter.missingDocs true
24
+
23
25
/--
24
26
A bitvector of the specified width.
25
27
@@ -34,9 +36,9 @@ structure BitVec (w : Nat) where
34
36
O(1), because we use `Fin` as the internal representation of a bitvector. -/
35
37
toFin : Fin (2 ^w)
36
38
37
- @[deprecated (since := "2024-04-12")]
38
- protected abbrev Std.BitVec := _root_. BitVec
39
-
39
+ /--
40
+ Bitvectors have decidable equality. This should be used via the instance `DecidableEq ( BitVec n)`.
41
+ -/
40
42
-- We manually derive the `DecidableEq` instances for `BitVec` because
41
43
-- we want to have builtin support for bit-vector literals, and we
42
44
-- need a name for this function to implement `canUnfoldAtMatcher` at `WHNF.lean`.
Original file line number Diff line number Diff line change @@ -28,6 +28,8 @@ https://github.com/mhk119/lean-smt/blob/bitvec/Smt/Data/Bitwise.lean.
28
28
29
29
-/
30
30
31
+ set_option linter.missingDocs true
32
+
31
33
open Nat Bool
32
34
33
35
namespace Bool
Original file line number Diff line number Diff line change @@ -8,6 +8,8 @@ import Init.Data.BitVec.Lemmas
8
8
import Init.Data.Nat.Lemmas
9
9
import Init.Data.Fin.Iterate
10
10
11
+ set_option linter.missingDocs true
12
+
11
13
namespace BitVec
12
14
13
15
/--
Original file line number Diff line number Diff line change @@ -12,6 +12,8 @@ import Init.Data.Nat.Lemmas
12
12
import Init.Data.Nat.Mod
13
13
import Init.Data.Int.Bitwise.Lemmas
14
14
15
+ set_option linter.missingDocs true
16
+
15
17
namespace BitVec
16
18
17
19
/--
You can’t perform that action at this time.
0 commit comments