src/HOL/Bali/DeclConcepts.thy
changeset 19564 d3e2f532459a
parent 16417 9bc16273c2d4
child 21765 89275a3ed7be
--- a/src/HOL/Bali/DeclConcepts.thy	Fri May 05 16:50:58 2006 +0200
+++ b/src/HOL/Bali/DeclConcepts.thy	Fri May 05 17:17:21 2006 +0200
@@ -1914,12 +1914,12 @@
 	   next
 	     case Some
 	     with dynM
-	     have termination: "?Termination"
+	     have "termination": "?Termination"
 	       by (auto)
 	     with Some dynM
 	     have "?Dynmethd_def dynC sig=Some dynM"
 	      by (auto simp add: dynmethd_dynC_def)
-	     with subclseq_super_statC statM dynM termination
+	     with subclseq_super_statC statM dynM "termination"
 	     show ?thesis
 	       by (auto simp add: dynmethd_def)
 	   qed