src/HOL/Code_Evaluation.thy
changeset 58334 7553a1bcecb7
parent 58310 91ea607a34d8
child 58350 919149921e46
--- a/src/HOL/Code_Evaluation.thy	Sat Sep 13 18:08:45 2014 +0200
+++ b/src/HOL/Code_Evaluation.thy	Sun Sep 14 22:59:30 2014 +0200
@@ -13,7 +13,7 @@
 
 subsubsection {* Terms and class @{text term_of} *}
 
-datatype "term" = dummy_term
+datatype (plugins only: code) "term" = dummy_term
 
 definition Const :: "String.literal \<Rightarrow> typerep \<Rightarrow> term" where
   "Const _ _ = dummy_term"
@@ -113,7 +113,7 @@
 
 end
 
-declare [[code drop: rec_term case_term size_term "size :: term \<Rightarrow> _" "HOL.equal :: term \<Rightarrow> _"
+declare [[code drop: rec_term case_term "HOL.equal :: term \<Rightarrow> _"
   "term_of :: typerep \<Rightarrow> _" "term_of :: term \<Rightarrow> _" "term_of :: String.literal \<Rightarrow> _"
   "term_of :: _ Predicate.pred \<Rightarrow> term" "term_of :: _ Predicate.seq \<Rightarrow> term"]]