diff -r 2bee5ca44ef5 -r bb5d3278f02e Quot/Examples/FSet.thy --- a/Quot/Examples/FSet.thy Mon Dec 07 21:53:50 2009 +0100 +++ b/Quot/Examples/FSet.thy Mon Dec 07 21:54:14 2009 +0100 @@ -427,5 +427,28 @@ apply (tactic {* lift_tac_fset @{context} @{thm list.cases(2)} 1 *}) done +lemma ttt: "((op @) x ((op #) e [])) = (((op #) e x))" +sorry +lemma "(FUNION x (INSERT e EMPTY)) = ((INSERT e x))" +apply (tactic {* lift_tac @{context} @{thm ttt} 1 *}) +done + +lemma ttt2: "(\e. ((op @) x ((op #) e []))) = (\e. ((op #) e x))" +sorry + +lemma "(\e. (FUNION x (INSERT e EMPTY))) = (\e. (INSERT e x))" +apply (tactic {* procedure_tac @{context} @{thm ttt2} 1 *}) +apply(tactic {* regularize_tac @{context} 1 *}) +defer +apply(tactic {* REPEAT_ALL_NEW (inj_repabs_tac_fset @{context}) 1*}) +(* apply(tactic {* clean_tac @{context} 1 *}) *) +sorry + +lemma ttt3: "(\x. ((op @) x ((op #) e []))) = (\x. ((op #) e x))" +sorry + +lemma "(\x. (FUNION x (INSERT e EMPTY))) = (\x. (INSERT e x))" +(* apply (tactic {* procedure_tac @{context} @{thm ttt3} 1 *}) *) +sorry end