thys/Spec.thy
changeset 293 1a4e5b94293b
parent 289 807acaf7f599
child 295 c6ec5f369037
--- a/thys/Spec.thy	Mon Sep 10 21:41:54 2018 +0100
+++ b/thys/Spec.thy	Sun Sep 30 12:02:04 2018 +0100
@@ -163,6 +163,7 @@
 
 lemma nullable_correctness:
   shows "nullable r  \<longleftrightarrow> [] \<in> (L r)"
+  apply(induct r)
 by (induct r) (auto simp add: Sequ_def) 
 
 lemma der_correctness: