src/HOL/List.thy
changeset 66836 4eb431c3f974
parent 66658 59acf5e73176
child 66847 e8282131ddf9
--- a/src/HOL/List.thy	Tue Oct 10 22:18:58 2017 +0100
+++ b/src/HOL/List.thy	Mon Oct 09 19:10:47 2017 +0200
@@ -6600,39 +6600,6 @@
   by (induction xs) simp_all
 
 
-subsection \<open>Transfer\<close>
-
-definition embed_list :: "nat list \<Rightarrow> int list" where
-"embed_list l = map int l"
-
-definition nat_list :: "int list \<Rightarrow> bool" where
-"nat_list l = nat_set (set l)"
-
-definition return_list :: "int list \<Rightarrow> nat list" where
-"return_list l = map nat l"
-
-lemma transfer_nat_int_list_return_embed: "nat_list l \<longrightarrow>
-    embed_list (return_list l) = l"
-  unfolding embed_list_def return_list_def nat_list_def nat_set_def
-  apply (induct l)
-  apply auto
-done
-
-lemma transfer_nat_int_list_functions:
-  "l @ m = return_list (embed_list l @ embed_list m)"
-  "[] = return_list []"
-  unfolding return_list_def embed_list_def
-  apply auto
-  apply (induct l, auto)
-  apply (induct m, auto)
-done
-
-(*
-lemma transfer_nat_int_fold1: "fold f l x =
-    fold (%x. f (nat x)) (embed_list l) x";
-*)
-
-
 subsection \<open>Code generation\<close>
 
 text\<open>Optional tail recursive version of @{const map}. Can avoid