(* Title: HOL/Induct/PropLog.thy Author: Tobias Nipkow Copyright 1994 TU Muenchen & University of Cambridge *) section ‹Meta-theory of propositional logic› theory PropLog imports Main begin text ‹ Datatype definition of propositional logic formulae and inductive definition of the propositional tautologies. Inductive definition of propositional logic. Soundness and completeness w.r.t.\ truth-tables. Prove: If ‹H ⊨ p› then ‹G ⊨ p› where ‹G ∈ Fin(H)› › subsection ‹The datatype of propositions›