Skip to content

Commit 41413d4

Browse files
committed
recover prettier proof
1 parent 05642c2 commit 41413d4

File tree

2 files changed

+3
-6
lines changed

2 files changed

+3
-6
lines changed

src/Init/Data/UInt/BasicAux.lean

Lines changed: 0 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -113,12 +113,10 @@ instance : Sub USize := ⟨USize.sub⟩
113113
instance : LT USize := ⟨USize.lt⟩
114114
instance : LE USize := ⟨USize.le⟩
115115

116-
set_option bootstrap.genMatcherCode false in
117116
@[extern "lean_usize_dec_lt"]
118117
def USize.decLt (a b : USize) : Decidable (a < b) :=
119118
inferInstanceAs (Decidable (a.toBitVec < b.toBitVec))
120119

121-
set_option bootstrap.genMatcherCode false in
122120
@[extern "lean_usize_dec_le"]
123121
def USize.decLe (a b : USize) : Decidable (a ≤ b) :=
124122
inferInstanceAs (Decidable (a.toBitVec ≤ b.toBitVec))

src/Std/Data/DHashMap/Internal/Index.lean

Lines changed: 3 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -56,10 +56,9 @@ cf. https://github.com/leanprover/lean4/issues/4157
5656
· exact h'
5757
· rw [USize.le_def, BitVec.le_def]
5858
change _ ≤ (_ % _)
59-
rw [Nat.mod_eq_of_lt h']
60-
rw [USize.toBitVec_eq_of_lt]
61-
· omega
62-
· cases usize_size_eq <;> omega
59+
rw [Nat.mod_eq_of_lt h', USize.ofNat, BitVec.toNat_ofNat, Nat.mod_eq_of_lt]
60+
. exact h
61+
· exact Nat.lt_of_le_of_lt h h'
6362
· exact Nat.lt_of_lt_of_le (USize.toNat_lt_size _) (Nat.le_of_not_lt h')⟩
6463

6564
end Std.DHashMap.Internal

0 commit comments

Comments
 (0)