Skip to content

Commit

Permalink
chore: add toint abs
Browse files Browse the repository at this point in the history
  • Loading branch information
bollu committed Oct 21, 2024
1 parent 6a110aa commit 1405f9c
Showing 1 changed file with 178 additions and 0 deletions.
178 changes: 178 additions & 0 deletions src/Init/Data/BitVec/Lemmas.lean
Original file line number Diff line number Diff line change
Expand Up @@ -2766,6 +2766,184 @@ theorem abs_cases (x : BitVec w) : x.abs =
by_cases hx : x.slt 0#w <;> by_cases hx' : x = intMin w <;> simp [hx, hx']


@[simp]
theorem toInt_of_length_zero (x : BitVec 0) : x.toInt = 0 := by
simp [BitVec.of_length_zero]


/-
Similar to toInt_eq_toNat_cond, but rewrites in terms of power of two manipulations,
instead of ugly `2 * x < 2^n`.
-/
@[simp]
theorem toInt_eq_toNat_cond' (x : BitVec n) (hn : n > 0) :
x.toInt =
if x.toNat < 2^(n - 1) then
(x.toNat : Int)
else
(x.toNat : Int) - (2^n : Nat) := by
rcases n with _ | n <;> try contradiction
simp only [gt_iff_lt, Nat.zero_lt_succ, Nat.add_one_sub_one] at *
rw [BitVec.toInt_eq_toNat_cond]
simp only [Nat.pow_succ, Int.natCast_mul, Int.Nat.cast_ofNat_Int]
by_cases hx : x.toNat < 2 ^ n
· simp [show 2 * x.toNat < 2 ^ n * 2 by omega, hx]
· simp [show ¬ 2 * x.toNat < 2^ n * 2 by omega, hx]

/-- info: 'BitVec.toInt_eq_toNat_cond'' depends on axioms: [propext, Quot.sound] -/
#guard_msgs in #print axioms BitVec.toInt_eq_toNat_cond'

-- TODO: make this the theorem, because this does not create 2^(w - 1)
-- nonsense.
-- TODO: make `msb` the simp normal form for checking if number is positive
-- or whatever.
@[bv_toNat] theorem msb_eq_decide' (x : BitVec w) :
BitVec.msb x = decide (2 ^ w ≤ 2 * x.toNat) := by
rw [x.msb_eq_getLsbD_last, x.getLsbD_last]
simp
rcases w with rfl | w <;> simp <;> omega


/-- info: 'BitVec.msb_eq_decide'' depends on axioms: [propext, Classical.choice, Quot.sound] -/
#guard_msgs in #print axioms BitVec.msb_eq_decide'

/-
Next thing we want to know: bounds on the value of `x.toInt`
-/
theorem toInt_bounds_of_msb_eq_false {x : BitVec n} (hmsb : x.msb = false) :
0 ≤ x.toInt ∧ 2 * x.toInt < 2^n := by
have := x.msb_eq_decide'
rw [hmsb] at this
simp only [false_eq_decide_iff, Nat.not_le] at this
rw [BitVec.toInt_eq_toNat_cond]
simp [this]
apply And.intro
· omega
· norm_cast

/--
info: 'BitVec.toInt_bounds_of_msb_eq_false' depends on axioms: [propext, Classical.choice, Quot.sound]
-/
#guard_msgs in #print axioms BitVec.toInt_bounds_of_msb_eq_false

theorem toInt_bounds_of_msb_eq_true {x : BitVec n} (hmsb : x.msb = true) :
-2^n ≤ x.toInt ∧ x.toInt < 0 := by
have := x.msb_eq_decide'
rw [hmsb] at this
simp only [true_eq_decide_iff] at this
rw [BitVec.toInt_eq_toNat_cond]
simp [show ¬ 2 * x.toNat < 2 ^ n by omega]
apply And.intro
· norm_cast
omega
· omega

/--
info: 'BitVec.toInt_bounds_of_msb_eq_true' depends on axioms: [propext, Classical.choice, Quot.sound]
-/
#guard_msgs in #print axioms BitVec.toInt_bounds_of_msb_eq_true

theorem toInt_intMin_eq_cases (n : Nat) : (BitVec.intMin n).toInt =
if n = 0 then 0 else - 2^(n - 1) := by
simp [BitVec.toInt_intMin]
rcases n with rfl | n
· simp
· simp
norm_cast
have : 2^n > 0 := by exact Nat.two_pow_pos n
have : 2^n < 2^(n + 1) := by
simp [Nat.pow_succ]
omega
rw [Nat.mod_eq_of_lt (by omega)]

/-- info: 'BitVec.toInt_intMin_eq_cases' depends on axioms: [propext, Quot.sound] -/
#guard_msgs in #print axioms BitVec.toInt_intMin_eq_cases

-- ### TOINT OF NEG
/--
Define the value of (BitVec.neg.toInt) as a case split
on whether `x` is intMin or not, and showing that when this
exception does not occur, the defn obeys what mathematics says it should
-/
theorem toInt_neg_eq_cases {x : BitVec n} :
(-x).toInt =
if x = intMin n
then x.toInt
else - x.toInt := by
by_cases hx : x = intMin n
· simp [hx]
· simp [hx]
rw [toInt_neg_of_ne_intMin hx]

/-- info: 'BitVec.toInt_neg_eq_cases' depends on axioms: [propext, Quot.sound] -/
#guard_msgs in #print axioms BitVec.toInt_neg_eq_cases

-- @[simp]
-- theorem Int.abs_neg (x : Int) : (-x).abs = x.abs := by
-- have hx : (-x < 0) ∨ (x = 0) ∨ (-x > 0) := by omega
-- rcases hx with hx | hx | hx
-- · rw [Int.abs_eq_neg (x := -x) hx, Int.neg_neg, Int.abs_eq_self (x := x) (by omega)]
-- · simp [hx]
-- · rw [Int.abs_eq_self (x := -x) (by omega), Int.abs_eq_neg (x := x) (by omega)]
--
--
-- /-- info: 'Int.abs_neg' depends on axioms: [propext, Quot.sound] -/
-- #guard_msgs in #print axioms Int.abs_neg


theorem abs_cases' (x : BitVec w) : x.abs =
if x.msb = true then
if x = BitVec.intMin w then (BitVec.intMin w) else -x
else x := by
· rw [BitVec.abs_def]
by_cases hx : x.msb = true <;> by_cases hx' : x = BitVec.intMin w <;> simp [hx, hx']

/-- info: 'BitVec.abs_cases'' depends on axioms: [propext, Quot.sound] -/
#guard_msgs in #print axioms BitVec.abs_cases'



theorem toInt_intMin_eq_twoPow (hn : 0 < n) : (intMin n).toInt = -2^(n - 1) := by
-- Delete our toInt_intMin from simp set.
rw [BitVec.toInt_intMin_eq_cases]
simp [show ¬ n = 0 by omega]

/-- info: 'BitVec.toInt_intMin_eq_twoPow' depends on axioms: [propext, Quot.sound] -/
#guard_msgs in #print axioms BitVec.toInt_intMin_eq_twoPow

theorem toInt_abs (x : BitVec w) :
x.abs.toInt = if x = (intMin w) then if w = 0 then 0 else - 2^(w - 1) else x.toInt.abs := by
rcases w with rfl | w
· simp
· simp only [gt_iff_lt, Nat.zero_lt_succ, Nat.add_one_ne_zero, ↓reduceIte]
rw [BitVec.abs_cases']
by_cases hx : x = intMin (w + 1)
· simp only [hx, reduceIte]
have := BitVec.msb_intMin (w := w + 1)
rw [this]
simp only [gt_iff_lt, Nat.zero_lt_succ, decide_True, ↓reduceIte]
rw [BitVec.toInt_intMin_eq_cases]
simp
· simp only [hx, reduceIte]
rcases hmsb : x.msb
· simp only [Bool.false_eq_true, ↓reduceIte]
have := BitVec.toInt_bounds_of_msb_eq_false hmsb
rw [Int.abs_eq_self]
omega
· simp only [reduceIte]
have hxbounds := BitVec.toInt_bounds_of_msb_eq_true hmsb
rw [BitVec.toInt_neg_eq_cases]
have hxneq : x.toInt ≠ (intMin (w + 1)).toInt := by
rw [BitVec.toInt_ne]
exact hx
rw [BitVec.toInt_intMin_eq_twoPow (by omega)] at hxneq
-- TODO: remove toInt_eq_toNat_cond from simp set.
simp only [hx, reduceIte]
rw [Int.abs_eq_neg (by omega)]

/-- info: 'BitVec.toInt_abs' depends on axioms: [propext, Classical.choice, Quot.sound] -/
#guard_msgs in #print axioms BitVec.toInt_abs

/-! ### Non-overflow theorems -/

/-- If `x.toNat * y.toNat < 2^w`, then the multiplication `(x * y)` does not overflow. -/
Expand Down

0 comments on commit 1405f9c

Please sign in to comment.