src/HOL/Library/Transitive_Closure_Table.thy
changeset 56922 d411a81b8356
parent 55419 8b7c7157fa11
child 58881 b9556a055632
--- a/src/HOL/Library/Transitive_Closure_Table.thy	Fri May 09 08:13:28 2014 +0200
+++ b/src/HOL/Library/Transitive_Closure_Table.thy	Fri May 09 08:13:36 2014 +0200
@@ -190,29 +190,4 @@
 
 code_pred rtranclp using rtranclp_eq_rtrancl_tab_nil [THEN iffD1] by fastforce
 
-subsection {* A simple example *}
-
-datatype ty = A | B | C
-
-inductive test :: "ty \<Rightarrow> ty \<Rightarrow> bool"
-where
-  "test A B"
-| "test B A"
-| "test B C"
-
-subsubsection {* Invoking with the predicate compiler and the generic code generator *}
-
-code_pred test .
-
-values "{x. test\<^sup>*\<^sup>* A C}"
-values "{x. test\<^sup>*\<^sup>* C A}"
-values "{x. test\<^sup>*\<^sup>* A x}"
-values "{x. test\<^sup>*\<^sup>* x C}"
-
-value "test\<^sup>*\<^sup>* A C"
-value "test\<^sup>*\<^sup>* C A"
-
-hide_type ty
-hide_const test A B C
-
 end
\ No newline at end of file