doc-src/TutorialI/Misc/pairs.thy
changeset 8745 13b32661dde4
child 9541 d17c0b34d5c8
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/doc-src/TutorialI/Misc/pairs.thy	Wed Apr 19 11:56:31 2000 +0200
@@ -0,0 +1,8 @@
+(*<*)
+theory pairs = Main:;
+term(*>*) "let (x,y) = f z in (y,x)";
+(*<*)
+term(*>*) "case xs of [] \\<Rightarrow> 0 | (x,y)#zs \\<Rightarrow> x+y"
+(**)(*<*)
+end
+(*>*)