Quot/Nominal/LamEx2.thy
changeset 1028 41fc4d3fc764
parent 1026 278253330b6a
child 1087 bb7f4457091a
equal deleted inserted replaced
1027:163d6917af62 1028:41fc4d3fc764
     2 imports "Nominal2_Atoms" "Nominal2_Eqvt" "Nominal2_Supp" "../QuotMain" "Abs" "../QuotProd"
     2 imports "Nominal2_Atoms" "Nominal2_Eqvt" "Nominal2_Supp" "../QuotMain" "Abs" "../QuotProd"
     3 begin
     3 begin
     4 
     4 
     5 
     5 
     6 (* lemmas that should be in Nominal \<dots>\<dots>must be cleaned *)
     6 (* lemmas that should be in Nominal \<dots>\<dots>must be cleaned *)
       
     7 (* Currently not used, still needed needed? *)
     7 lemma supp_finite_set:
     8 lemma supp_finite_set:
     8   fixes S::"atom set"
     9   fixes S::"atom set"
     9   assumes "finite S"
    10   assumes "finite S"
    10   shows "supp S = S"
    11   shows "supp S = S"
    11   apply(rule finite_supp_unique)
    12   apply(rule finite_supp_unique)