LamEx.thy
changeset 203 7384115df9fd
parent 201 1ac36993cc71
child 217 9cc87d02190a
child 218 df05cd030d2f
--- a/LamEx.thy	Tue Oct 27 11:43:02 2009 +0100
+++ b/LamEx.thy	Tue Oct 27 14:14:30 2009 +0100
@@ -17,8 +17,11 @@
 | a3: "\<lbrakk>t \<approx> ([(a,b)]\<bullet>s); a\<sharp>s\<rbrakk> \<Longrightarrow> rLam a t \<approx> rLam b s"
 
 quotient lam = rlam / alpha
+apply -
 sorry
 
+print_quotients
+
 local_setup {*
   make_const_def @{binding Var} @{term "rVar"} NoSyn @{typ "rlam"} @{typ "lam"} #> snd #>
   make_const_def @{binding App} @{term "rApp"} NoSyn @{typ "rlam"} @{typ "lam"} #> snd #>