src/HOL/HOLCF/Library/Char_Discrete.thy
changeset 58880 0baae4311a9f
parent 42151 4da4fc77664b
child 62175 8ffc4d0e652d
equal deleted inserted replaced
58879:143c85e3cdb5 58880:0baae4311a9f
     1 (*  Title:      HOL/HOLCF/Library/Char_Discrete.thy
     1 (*  Title:      HOL/HOLCF/Library/Char_Discrete.thy
     2     Author:     Brian Huffman
     2     Author:     Brian Huffman
     3 *)
     3 *)
     4 
     4 
     5 header {* Discrete cpo instance for 8-bit char type *}
     5 section {* Discrete cpo instance for 8-bit char type *}
     6 
     6 
     7 theory Char_Discrete
     7 theory Char_Discrete
     8 imports HOLCF
     8 imports HOLCF
     9 begin
     9 begin
    10 
    10