src/HOL/Word/Bit_Representation.thy
changeset 46000 871bdab23f5c
parent 45999 cce7e6197a46
child 46001 0b562d564d5f
equal deleted inserted replaced
45999:cce7e6197a46 46000:871bdab23f5c
   721   zmod_uminus' [symmetric]
   721   zmod_uminus' [symmetric]
   722   mod_add_left_eq [where b = "1::int"]
   722   mod_add_left_eq [where b = "1::int"]
   723   zmod_zsub_left_eq [where b = "1"]
   723   zmod_zsub_left_eq [where b = "1"]
   724 
   724 
   725 lemmas bintr_arith1s =
   725 lemmas bintr_arith1s =
   726   brdmod1s' [where c="2^n::int", folded pred_def succ_def bintrunc_mod2p] for n
   726   brdmod1s' [where c="2^n::int", folded bintrunc_mod2p] for n
   727 lemmas bintr_ariths =
   727 lemmas bintr_ariths =
   728   brdmods' [where c="2^n::int", folded pred_def succ_def bintrunc_mod2p] for n
   728   brdmods' [where c="2^n::int", folded bintrunc_mod2p] for n
   729 
   729 
   730 lemmas m2pths = pos_mod_sign pos_mod_bound [OF zless2p]
   730 lemmas m2pths = pos_mod_sign pos_mod_bound [OF zless2p]
   731 
   731 
   732 lemma bintr_ge0: "(0 :: int) <= number_of (bintrunc n w)"
   732 lemma bintr_ge0: "(0 :: int) <= number_of (bintrunc n w)"
   733   by (simp add : no_bintr m2pths)
   733   by (simp add : no_bintr m2pths)