changeset 44890 | 22f665a2e91c |
parent 43973 | a907e541b127 |
child 45169 | 4baa475a51e6 |
--- a/src/HOL/Library/Transitive_Closure_Table.thy Sun Sep 11 22:56:05 2011 +0200 +++ b/src/HOL/Library/Transitive_Closure_Table.thy Mon Sep 12 07:55:43 2011 +0200 @@ -189,7 +189,7 @@ declare rtranclp_eq_rtrancl_tab_nil[THEN iffD2, code_pred_intro] -code_pred rtranclp using rtranclp_eq_rtrancl_tab_nil [THEN iffD1] by fastsimp +code_pred rtranclp using rtranclp_eq_rtrancl_tab_nil [THEN iffD1] by fastforce subsection {* A simple example *}