src/HOL/Induct/PropLog.thy
changeset 58889 5b7a9633cfa8
parent 58310 91ea607a34d8
child 60530 44f9873d6f6f
equal deleted inserted replaced
58888:9537bf1c4853 58889:5b7a9633cfa8
     1 (*  Title:      HOL/Induct/PropLog.thy
     1 (*  Title:      HOL/Induct/PropLog.thy
     2     Author:     Tobias Nipkow
     2     Author:     Tobias Nipkow
     3     Copyright   1994  TU Muenchen & University of Cambridge
     3     Copyright   1994  TU Muenchen & University of Cambridge
     4 *)
     4 *)
     5 
     5 
     6 header {* Meta-theory of propositional logic *}
     6 section {* Meta-theory of propositional logic *}
     7 
     7 
     8 theory PropLog imports Main begin
     8 theory PropLog imports Main begin
     9 
     9 
    10 text {*
    10 text {*
    11   Datatype definition of propositional logic formulae and inductive
    11   Datatype definition of propositional logic formulae and inductive