diff -r 18efe191bd5f -r c29146dc14f1 src/HOL/Nominal/Examples/CR.thy --- a/src/HOL/Nominal/Examples/CR.thy Wed Nov 15 15:39:22 2006 +0100 +++ b/src/HOL/Nominal/Examples/CR.thy Wed Nov 15 16:23:55 2006 +0100 @@ -225,7 +225,7 @@ show ?case proof (simp) have f: "\c::name. c\(pi\a,pi\s1,pi\s2,x)" - by (rule at_exists_fresh[OF at_name_inst], simp add: fs_name1) + by (rule exists_fresh', simp add: fs_name1) then obtain c::"name" where f1: "c\(pi\a)" and f2: "c\x" and f3: "c\(pi\s1)" and f4: "c\(pi\s2)" by (force simp add: fresh_prod fresh_atm) @@ -243,7 +243,7 @@ show ?case proof (simp add: subst_eqvt) have f: "\c::name. c\(pi\a,pi\s1,pi\s2,x)" - by (rule at_exists_fresh[OF at_name_inst], simp add: fs_name1) + by (rule exists_fresh', simp add: fs_name1) then obtain c::"name" where f1: "c\(pi\a)" and f2: "c\x" and f3: "c\(pi\s1)" and f4: "c\(pi\s2)" by (force simp add: fresh_prod fresh_atm) @@ -320,7 +320,7 @@ show ?case proof (simp) have f: "\c::name. c\(pi\a,pi\t1,pi\t2,x)" - by (rule at_exists_fresh[OF at_name_inst], simp add: fs_name1) + by (rule exists_fresh', simp add: fs_name1) then obtain c::"name" where f1: "c\(pi\a)" and f2: "c\x" and f3: "c\(pi\t1)" and f4: "c\(pi\t2)" by (force simp add: fresh_prod fresh_atm) @@ -342,7 +342,7 @@ show ?case proof (simp) have f: "\c::name. c\(pi\a,pi\t1,pi\t2,pi\s1,pi\s2,x)" - by (rule at_exists_fresh[OF at_name_inst], simp add: fs_name1) + by (rule exists_fresh', simp add: fs_name1) then obtain c::"name" where f1: "c\(pi\a)" and f2: "c\x" and f3: "c\(pi\t1)" and f4: "c\(pi\t2)" by (force simp add: fresh_prod at_fresh[OF at_name_inst])