doc-src/TutorialI/Misc/consts.thy
author paulson
Tue, 05 Sep 2000 13:12:00 +0200
changeset 9843 cc8aa63bdad6
parent 8745 13b32661dde4
permissions -rw-r--r--
tidied, proving gcd_greatest_iff and using induct_tac

(*<*)theory "consts" = Main:;
(*>*)consts nand :: gate
            exor :: gate(*<*)
end
(*>*)