src/HOL/Import/Import_Setup.thy
author blanchet
Mon, 21 May 2012 10:39:31 +0200
changeset 47944 e6b51fab96f7
parent 47258 880e587eee9f
child 48891 c0eafbd55de3
permissions -rw-r--r--
added helper -- cf. SET616^5

(*  Title:      HOL/Import/Import_Setup.thy
    Author:     Cezary Kaliszyk, University of Innsbruck
    Author:     Alexander Krauss, QAware GmbH
*)

header {* Importer machinery and required theorems *}

theory Import_Setup
imports "~~/src/HOL/Parity" "~~/src/HOL/Fact"
keywords
    "import_type_map" :: thy_decl and "import_const_map" :: thy_decl and
    "import_file" :: thy_decl
uses "import_data.ML" ("import_rule.ML")
begin

lemma light_ex_imp_nonempty:
  "P t \<Longrightarrow> \<exists>x. x \<in> Collect P"
  by auto

lemma typedef_hol2hollight:
  assumes a: "type_definition Rep Abs (Collect P)"
  shows "Abs (Rep a) = a \<and> P r = (Rep (Abs r) = r)"
  by (metis type_definition.Rep_inverse type_definition.Abs_inverse
      type_definition.Rep a mem_Collect_eq)

lemma ext2:
  "(\<And>x. f x = g x) \<Longrightarrow> f = g"
  by auto

use "import_rule.ML"

end