(* Title: Containers/Examples/TwoSat_Ex.thy Author: Andreas Lochbihler, ETH Zurich Author: Peter Lammich, TU Munich *) section ‹Formalisation of 2SAT independent of an implementation› theory TwoSat_Ex imports Main "HOL-Library.Uprod" "Deriving.Compare_Instances" begin type_synonym var = nat