FSet.thy
changeset 496 8f1bf5266ebc
parent 495 76fa93b1fe8b
child 498 e7bb6bbe7576
equal deleted inserted replaced
495:76fa93b1fe8b 496:8f1bf5266ebc
   479 
   479 
   480 lemma "fset_case (f1::'t) f2 (INSERT a xa) = f2 a xa"
   480 lemma "fset_case (f1::'t) f2 (INSERT a xa) = f2 a xa"
   481 apply (tactic {* lift_tac_fset @{context} @{thm list.cases(2)} 1 *})
   481 apply (tactic {* lift_tac_fset @{context} @{thm list.cases(2)} 1 *})
   482 done
   482 done
   483 
   483 
       
   484 ML {* qconsts_lookup @{theory} "EMPTY" *}
       
   485 thm EMPTY_def
       
   486 
       
   487 
   484 end
   488 end