src/ZF/Induct/PropLog.thy
changeset 20503 503ac4c5ef91
parent 18415 eb68dc98bda2
child 24893 b8ef7afe3a6b
equal deleted inserted replaced
20502:08d227db6c74 20503:503ac4c5ef91
   325   -- {* A semantic analogue of the Deduction Theorem *}
   325   -- {* A semantic analogue of the Deduction Theorem *}
   326   by (simp add: logcon_def)
   326   by (simp add: logcon_def)
   327 
   327 
   328 lemma completeness:
   328 lemma completeness:
   329      "H \<in> Fin(propn) ==> p \<in> propn \<Longrightarrow> H |= p \<Longrightarrow> H |- p"
   329      "H \<in> Fin(propn) ==> p \<in> propn \<Longrightarrow> H |= p \<Longrightarrow> H |- p"
   330   apply (induct fixing: p set: Fin)
   330   apply (induct arbitrary: p set: Fin)
   331    apply (safe intro!: completeness_0)
   331    apply (safe intro!: completeness_0)
   332   apply (rule weaken_left_cons [THEN thms_MP])
   332   apply (rule weaken_left_cons [THEN thms_MP])
   333    apply (blast intro!: logcon_Imp propn.intros)
   333    apply (blast intro!: logcon_Imp propn.intros)
   334   apply (blast intro: propn_Is)
   334   apply (blast intro: propn_Is)
   335   done
   335   done