Quot/Examples/IntEx.thy
changeset 835 c4fa87dd0208
parent 833 129caba33c03
child 854 5961edda27d7
--- a/Quot/Examples/IntEx.thy	Mon Jan 11 01:03:34 2010 +0100
+++ b/Quot/Examples/IntEx.thy	Mon Jan 11 11:51:19 2010 +0100
@@ -199,6 +199,8 @@
 apply simp
 done
 
+
+term foldl
 lemma "foldl PLUS x [] = x"
 apply(lifting ho_tst)
 done