src/HOL/Types_To_Sets/Types_To_Sets.thy
author wenzelm
Fri, 23 Nov 2018 16:43:11 +0100
changeset 69334 6b49700da068
parent 68428 46beee72fb66
child 69605 a96320074298
permissions -rw-r--r--
clarified font_domain: strict excludes e.g. space character;

(*  Title:      HOL/Types_To_Sets/Types_To_Sets.thy
    Author:     Ondřej Kunčar, TU München
*)

section \<open>From Types to Sets\<close>

text \<open>This theory extends Isabelle/HOL's logic by two new inference rules
  to allow translation of types to sets as described in
  O. Kunčar, A. Popescu: From Types to Sets by Local Type Definitions in Higher-Order Logic
  available at https://www21.in.tum.de/~kuncar/documents/kuncar-popescu-t2s2016-extended.pdf.\<close>

theory Types_To_Sets
  imports Main
begin

subsection \<open>Rules\<close>

text\<open>The following file implements the Local Typedef Rule (LT) and extends the logic by the rule.\<close>
ML_file "local_typedef.ML"

text\<open>The following file implements the Unoverloading Rule (UO) and extends the logic by the rule.\<close>
ML_file "unoverloading.ML"

text\<open>The following file implements a derived rule that internalizes type class annotations.\<close>
ML_file "internalize_sort.ML"

text\<open>The following file provides some automation to unoverload and internalize the parameters o
  the sort constraints of a type variable.\<close>
ML_file \<open>unoverload_type.ML\<close>

end