src/ZF/Induct/Comb.thy
changeset 46900 73555abfa267
parent 46822 95f1e700b712
child 58623 2db1df2c8467
--- a/src/ZF/Induct/Comb.thy	Tue Mar 13 14:17:42 2012 +0100
+++ b/src/ZF/Induct/Comb.thy	Tue Mar 13 14:44:16 2012 +0100
@@ -114,8 +114,6 @@
 
 inductive_cases Ap_E [elim!]: "p\<bullet>q \<in> comb"
 
-declare comb.intros [intro!]
-
 
 subsection {* Results about Contraction *}
 
@@ -189,13 +187,13 @@
 text {* Counterexample to the diamond property for @{text "-1->"}. *}
 
 lemma KIII_contract1: "K\<bullet>I\<bullet>(I\<bullet>I) -1-> I"
-  by (blast intro: comb.intros contract.K comb_I)
+  by (blast intro: comb_I)
 
 lemma KIII_contract2: "K\<bullet>I\<bullet>(I\<bullet>I) -1-> K\<bullet>I\<bullet>((K\<bullet>I)\<bullet>(K\<bullet>I))"
-  by (unfold I_def) (blast intro: comb.intros contract.intros)
+  by (unfold I_def) (blast intro: contract.intros)
 
 lemma KIII_contract3: "K\<bullet>I\<bullet>((K\<bullet>I)\<bullet>(K\<bullet>I)) -1-> I"
-  by (blast intro: comb.intros contract.K comb_I)
+  by (blast intro: comb_I)
 
 lemma not_diamond_contract: "\<not> diamond(contract)"
   apply (unfold diamond_def)