Correctness.thy
changeset 161 f1d82f6c05a3
parent 160 83da37e8b1d2
child 170 def87c589516
--- a/Correctness.thy	Fri Apr 21 20:17:13 2017 +0800
+++ b/Correctness.thy	Tue Apr 25 14:05:57 2017 +0100
@@ -1287,6 +1287,9 @@
 
 definition "up_to s t = map (\<lambda> t'. t'@s) (postfixes t)"
 
+
+
+
 definition "occs' Q tt = length (filter Q (postfixes tt))"
 
 lemma occs'_nil [simp]: "occs' Q [] = 0"