no need thanks to "Code.abort"
authorblanchet
Wed, 18 Sep 2013 17:36:47 +0200
changeset 53698 e1b039dada7b
parent 53697 221ec353bcc5
child 53699 7d32f33d340d
no need thanks to "Code.abort"
src/HOL/BNF/BNF_FP_Base.thy
--- a/src/HOL/BNF/BNF_FP_Base.thy	Wed Sep 18 16:44:19 2013 +0200
+++ b/src/HOL/BNF/BNF_FP_Base.thy	Wed Sep 18 17:36:47 2013 +0200
@@ -13,11 +13,6 @@
 imports BNF_Comp BNF_Ctr_Sugar
 begin
 
-definition code_unspec :: "(unit \<Rightarrow> 'a) \<Rightarrow> 'a" where
-[code del]: "code_unspec f = f ()"
-
-code_abort code_unspec
-
 lemma mp_conj: "(P \<longrightarrow> Q) \<and> R \<Longrightarrow> P \<Longrightarrow> R \<and> Q"
 by auto