(* Copyright 2021, Data61, CSIRO (ABN 41 687 119 230) SPDX-License-Identifier: CC-BY-SA-4.0 *) theory Style_pre imports Main begin text \ This a helper theory for Style.thy. \ typedecl type_foo typedecl type_bar definition valid :: "'a \ 'b \ 'c \ bool" ("\_\/ _ /\_\") where "\P\ f \Q\ \ undefined" definition pred_conj :: "('a \ bool) \ ('a \ bool) \ ('a \ bool)" (infixl "and" 35) where "pred_conj P Q \ \x. P x \ Q x" end