src/HOL/Induct/PropLog.thy
changeset 17589 58eeffd73be1
parent 16563 a92f96951355
child 18260 5597cfcecd49
--- a/src/HOL/Induct/PropLog.thy	Thu Sep 22 23:55:42 2005 +0200
+++ b/src/HOL/Induct/PropLog.thy	Thu Sep 22 23:56:15 2005 +0200
@@ -236,12 +236,12 @@
 apply (rule hyps_subset [THEN hyps_finite [THEN finite_subset_induct]])
  apply (simp add: sat_thms_p, safe)
  txt{*Case @{text"hyps p t-insert(#v,Y) |- p"} *}
- apply (rules intro: thms_excluded_middle_rule 
+ apply (iprover intro: thms_excluded_middle_rule 
 		     insert_Diff_same [THEN weaken_left]
                      insert_Diff_subset2 [THEN weaken_left] 
                      hyps_Diff [THEN Diff_weaken_left])
 txt{*Case @{text"hyps p t-insert(#v -> false,Y) |- p"} *}
- apply (rules intro: thms_excluded_middle_rule 
+ apply (iprover intro: thms_excluded_middle_rule 
 		     insert_Diff_same [THEN weaken_left]
                      insert_Diff_subset2 [THEN weaken_left] 
                      hyps_insert [THEN Diff_weaken_left])
@@ -260,7 +260,7 @@
 theorem completeness [rule_format]: "finite H ==> \<forall>p. H |= p --> H |- p"
 apply (erule finite_induct)
  apply (blast intro: completeness_0)
-apply (rules intro: sat_imp thms.H insertI1 weaken_left_insert [THEN thms.MP])
+apply (iprover intro: sat_imp thms.H insertI1 weaken_left_insert [THEN thms.MP])
 done
 
 theorem syntax_iff_semantics: "finite H ==> (H |- p) = (H |= p)"