src/HOL/Predicate_Compile_Examples/Predicate_Compile_Tests.thy
changeset 39657 5e57675b7e40
parent 39655 8ad7fe9d6f0b
child 39762 02fb709ab3cb
--- a/src/HOL/Predicate_Compile_Examples/Predicate_Compile_Tests.thy	Thu Sep 23 14:50:18 2010 +0200
+++ b/src/HOL/Predicate_Compile_Examples/Predicate_Compile_Tests.thy	Thu Sep 23 17:22:44 2010 +0200
@@ -1327,10 +1327,10 @@
 text {* The global introduction rules must be redeclared as introduction rules and then 
   one could invoke code_pred. *}
 
-declare A.hd_predicate_in_locale.intros [unfolded Predicate.eq_is_eq[symmetric], code_pred_intro]
+declare A.hd_predicate_in_locale.intros [code_pred_intro]
 
 code_pred (expected_modes: i => i => i => bool, i => i => o => bool) A.hd_predicate_in_locale
-unfolding eq_is_eq by (auto elim: A.hd_predicate_in_locale.cases)
+by (auto elim: A.hd_predicate_in_locale.cases)
     
 interpretation A partial_hd .
 thm hd_predicate_in_locale.intros