src/HOL/Predicate_Compile_Examples/Predicate_Compile_Tests.thy
changeset 47433 07f4bf913230
parent 47108 2a1953f0d20d
child 51143 0a2371e7ced3
--- a/src/HOL/Predicate_Compile_Examples/Predicate_Compile_Tests.thy	Tue Apr 03 08:55:06 2012 +0200
+++ b/src/HOL/Predicate_Compile_Examples/Predicate_Compile_Tests.thy	Tue Apr 03 17:26:30 2012 +0900
@@ -1027,8 +1027,8 @@
   (o * o => bool) => i * i => bool) [inductify] converse .
 
 thm converse.equation
-code_pred [inductify] rel_comp .
-thm rel_comp.equation
+code_pred [inductify] relcomp .
+thm relcomp.equation
 code_pred [inductify] Image .
 thm Image.equation
 declare singleton_iff[code_pred_inline]