Quot/Examples/FSet.thy
changeset 609 6ce4f274b0fa
parent 600 5d932e7a856c
child 611 bb5d3278f02e
equal deleted inserted replaced
608:678315da994e 609:6ce4f274b0fa
   434 
   434 
   435 lemma "fset_case (f1::'t) f2 (INSERT a xa) = f2 a xa"
   435 lemma "fset_case (f1::'t) f2 (INSERT a xa) = f2 a xa"
   436 apply (tactic {* lift_tac_fset @{context} @{thm list.cases(2)} 1 *})
   436 apply (tactic {* lift_tac_fset @{context} @{thm list.cases(2)} 1 *})
   437 done
   437 done
   438 
   438 
       
   439 lemma ttt: "((op @) x ((op #) e [])) = (((op #) e x))"
       
   440 sorry
       
   441 lemma "(FUNION x (INSERT e EMPTY)) = ((INSERT e x))"
       
   442 apply (tactic {* lift_tac @{context} @{thm ttt} 1 *})
       
   443 done
       
   444 
       
   445 lemma ttt2: "(\<lambda>e. ((op @) x ((op #) e []))) = (\<lambda>e. ((op #) e x))"
       
   446 sorry
       
   447 
       
   448 lemma "(\<lambda>e. (FUNION x (INSERT e EMPTY))) = (\<lambda>e. (INSERT e x))"
       
   449 apply (tactic {* procedure_tac @{context} @{thm ttt2} 1 *})
       
   450 apply(tactic {* regularize_tac @{context} 1 *})
       
   451 defer
       
   452 apply(tactic {* REPEAT_ALL_NEW (inj_repabs_tac_fset @{context}) 1*})
       
   453 (* apply(tactic {* clean_tac @{context} 1 *}) *)
       
   454 sorry
       
   455 
       
   456 lemma ttt3: "(\<lambda>x. ((op @) x ((op #) e []))) = (\<lambda>x. ((op #) e x))"
       
   457 sorry
       
   458 
       
   459 lemma "(\<lambda>x. (FUNION x (INSERT e EMPTY))) = (\<lambda>x. (INSERT e x))"
       
   460 (* apply (tactic {* procedure_tac @{context} @{thm ttt3} 1 *}) *)
       
   461 sorry
   439 
   462 
   440 end
   463 end