src/HOL/ex/BinEx.thy
author paulson
Mon, 16 Nov 1998 10:37:54 +0100
changeset 5866 de6a1856c74a
parent 5545 9117a0e2bf31
child 6920 c912740c3545
permissions -rw-r--r--
removed the reference to mesontest2.ML, itself now deleted

(*  Title:      HOL/ex/BinEx.thy
    ID:         $Id$
    Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
    Copyright   1998  University of Cambridge

Definition of normal form for proving that binary arithmetic on
ormalized operands yields normalized results.

Normal means no leading 0s on positive numbers and no leading 1s on negatives.
*)

BinEx = Bin +

consts normal :: bin set
  
inductive "normal"
  intrs 

    Pls  "Pls: normal"

    Min  "Min: normal"

    BIT_F  "[| w: normal; w ~= Pls |] ==> w BIT False : normal"

    BIT_T  "[| w: normal; w ~= Min |] ==> w BIT True : normal"

end