src/HOL/ex/Word_Type.thy
changeset 64113 86efd3d4dc98
parent 64015 c9f3a94cb825
child 64114 45e065eea984
--- a/src/HOL/ex/Word_Type.thy	Sat Oct 08 17:30:19 2016 +0200
+++ b/src/HOL/ex/Word_Type.thy	Sat Oct 08 14:09:53 2016 +0200
@@ -9,21 +9,6 @@
     "~~/src/HOL/Library/Type_Length"
 begin
 
-subsection \<open>Compact syntax for types with a length\<close>
-
-syntax "_type_length" :: "type \<Rightarrow> nat" ("(1LENGTH/(1'(_')))")
-
-translations "LENGTH('a)" \<rightharpoonup>
-  "CONST len_of (CONST Pure.type :: 'a itself)"
-
-print_translation \<open>
-  let
-    fun len_of_itself_tr' ctxt [Const (@{const_syntax Pure.type}, Type (_, [T]))] =
-      Syntax.const @{syntax_const "_type_length"} $ Syntax_Phases.term_of_typ ctxt T
-  in [(@{const_syntax len_of}, len_of_itself_tr')] end
-\<close>
-
-
 subsection \<open>Truncating bit representations of numeric types\<close>
 
 class semiring_bits = semiring_div_parity +