# HG changeset patch # User Cezary Kaliszyk # Date 1260217549 -3600 # Node ID 6ce4f274b0fab0b4571e232840d57daaaa455fc9 # Parent 678315da994ee61046e6b46fcd447e22c22bde86 3 lambda examples in FSet. In the last one regularize_term fails. diff -r 678315da994e -r 6ce4f274b0fa Quot/Examples/FSet.thy --- a/Quot/Examples/FSet.thy Mon Dec 07 21:21:57 2009 +0100 +++ b/Quot/Examples/FSet.thy Mon Dec 07 21:25:49 2009 +0100 @@ -436,5 +436,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