doc-src/TutorialI/Misc/consts.thy
author wenzelm
Sat, 18 Nov 2000 19:46:48 +0100
changeset 10491 e4a408728012
parent 8745 13b32661dde4
permissions -rw-r--r--
quot_cond_function: simplified, support conditional definition;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
8745
13b32661dde4 I wonder which files i forgot.
nipkow
parents:
diff changeset
     1
(*<*)theory "consts" = Main:;
13b32661dde4 I wonder which files i forgot.
nipkow
parents:
diff changeset
     2
(*>*)consts nand :: gate
13b32661dde4 I wonder which files i forgot.
nipkow
parents:
diff changeset
     3
            exor :: gate(*<*)
13b32661dde4 I wonder which files i forgot.
nipkow
parents:
diff changeset
     4
end
13b32661dde4 I wonder which files i forgot.
nipkow
parents:
diff changeset
     5
(*>*)